lean2/tests/lean/simp27.lean.expected.out

14 lines
438 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Assumed: a
Assumed: b
Assumed: f
Assumed: g
λ x x2 : , (∀ y : , g y = x) → x > x2 + x
funext (λ x : ,
funext (λ x2 : ,
imp_congr
(refl (∀ y : , g y = x))
(λ C::3 : ∀ y : , g y = x,
congr (congr2 Nat::gt (C::3 (a + x + b))) (congr2 (Nat::add x2) (C::3 x)))))