lean2/tests/lean/print_ax2.lean.expected.out

2 lines
221 B
Text

funext : ∀ {A : Type} {B : A → Type} {f g : Π (a : A), B a}, (∀ (a : A), f a = g a) → f = g
strong_indefinite_description : Π {A : Type} (P : A → Prop), nonempty A → { (x : A) | (∃ (x : A), P x) → P x }