2015-07-29 00:14:51 +00:00
|
|
|
|
quot.sound : ∀ {A : Type} [s : setoid A] {a b : A}, setoid.r a b → quot.mk a = quot.mk b
|
2015-04-01 22:09:00 +00:00
|
|
|
|
em : ∀ (a : Prop), a ∨ ¬a
|
2015-07-29 00:14:51 +00:00
|
|
|
|
propext : ∀ {a b : Prop}, (a ↔ b) → a = b
|
2015-06-10 23:26:32 +00:00
|
|
|
|
strong_indefinite_description : Π {A : Type} (P : A → Prop), nonempty A → { (x : A)| Exists P → P x}
|