theory Propositions imports MLTT.Prelude Equivalence begin definition isProp where "isProp A \ \x y: A. x =\<^bsub>A\<^esub> y" definition isSet where "isSet A \ \x y: A. \p q: x =\<^bsub>A\<^esub> y. p =\<^bsub>x =\<^bsub>A\<^esub> y\<^esub> q" Theorem isProp_Top: "isProp \" unfolding isProp_def by (intros, elims, refl) Theorem isProp_Bot: "isProp \" unfolding isProp_def by (intros, elim) end