Martin Escardo

\begin{code}

{-# OPTIONS --safe --without-K #-}

module Notation.index where

import Notation.CanonicalMap
import Notation.General
import Notation.Order
import Notation.UnderlyingType

\end{code}