lean2/tests/lean/simp25.lean.expected.out

11 lines
352 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Assumed: a
Assumed: b
Assumed: f
λ x : , x = 1 ∧ f (λ y z : , y + z > 1)
funext (λ x : ,
and_congrr
(λ C::2 : f (λ y z : , y + z > x), refl (x = 1))
(λ C::9 : x = 1, congr2 f (funext (λ y : , funext (λ z : , congr2 (Nat::gt (y + z)) C::9)))))