theory Propositions imports MLTT.Prelude Equivalence begin Definition isProp: ":= \x y: A. x = y" where "A: U i" by typechk Definition isSet: ":=\x y: A. \p q: x = y. p = q" where "A: U i" by typechk Theorem isProp_Top: "isProp \" unfolding isProp_def by (intros, elims, refl) Theorem isProp_Bot: "isProp \" unfolding isProp_def by (intros, elim) end