Our Spartan (intensional) Martin-LΓΆf type theory has the empty type β
,
the unit type π, two-point-type π, natural numbers β, product types Ξ ,
sum types Ξ£ (and hence binary product types _Γ_), sum types _+_,
identity types _οΌ_, and universes π€, π₯, π¦, ....
\begin{code}
{-# OPTIONS --safe --without-K #-}
module MLTT.Spartan where
open import MLTT.Empty public
open import MLTT.Unit public
open import MLTT.Two public
open import MLTT.NaturalNumbers public
open import MLTT.Plus public
open import MLTT.Pi public
open import MLTT.Sigma public
open import MLTT.Universes public
open import MLTT.Id public
open import Notation.General public
\end{code}