lean2/tests/lean/nested1.lean.expected.out

9 lines
392 B
Text
Raw Normal View History

definition test.foo.prf [irreducible] : ∀ (x : ), 0 < succ (succ x) :=
λ (x : ), lt.step (zero_lt_succ x)
definition test.bla : :=
λ (a : ), foo (succ (succ a)) (foo.prf a)
definition test.bla : :=
λ (a : ), test.foo (succ (succ a)) (test.foo.prf a)
definition test.foo.prf : ∀ (x : ), 0 < succ (succ x) :=
λ (x : ), lt.step (zero_lt_succ x)