c45c1748d8
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
12 lines
569 B
Text
12 lines
569 B
Text
Set: pp::colors
|
||
Set: pp::unicode
|
||
Assumed: a
|
||
Assumed: b
|
||
λ x : ℕ, x = a
|
||
funext (λ x : ℕ, trans (imp_congr (eq_id a) (λ H : ⊤, refl (x = a))) (imp_truel (x = a)))
|
||
λ x : ℕ, ⊤
|
||
funext (λ x : ℕ, trans (imp_congr (refl (x = a)) (λ H : x = a, eq_id x)) (imp_truer (x = a)))
|
||
λ x : ℕ, ⊤
|
||
funext (λ x : ℕ, trans (imp_congr (congr2 (eq x) (Nat::add_zeror a)) (λ H : x = a, eq_id a)) (imp_truer (x = a)))
|
||
λ x : ℕ, a = 1 → x > 1
|
||
funext (λ x : ℕ, imp_congr (congr1 (congr2 eq (Nat::add_zeror a)) 1) (λ C::2 : a = 1, congr2 (Nat::gt x) C::2))
|