lean2/tests/lean/nested2.lean.expected.out

16 lines
849 B
Text
Raw Normal View History

definition bla : :=
λ (a : ), foo (succ (succ a)) (bla_2 a)
definition bla_1 : ∀ (x : ), 0 < succ x :=
λ (x : ), zero_lt_succ x
definition bla_2 : ∀ (x : ), 0 < succ (succ x) :=
λ (x : ), lt.step (bla_1 x)
definition test_1 [irreducible] : ∀ (x : ), 0 < succ x :=
λ (x : ), zero_lt_succ x
definition test_2 [reducible] : ∀ (x : ), 0 < succ (succ x) :=
λ (x : ), lt.step (test_1 x)
definition tst_1 : ∀ (x : Type.{l_1}) (x_1 : x) (x_2 : list.{l_1} x),
x_1 :: x_2 = nil.{l_1} → list.no_confusion_type.{0 l_1} false (x_1 :: x_2) nil.{l_1} :=
λ (x : Type.{l_1}) (x_1 : x) (x_2 : list.{l_1} x), list.no_confusion.{0 l_1}
definition tst : Π {A : Type.{l_1}}, A → list.{l_1} A → bool :=
λ (A : Type.{l_1}) (a : A) (l : list.{l_1} A), voo.{(max 1 l_1)} (a :: l) nil.{l_1} (tst_1.{l_1} A a l)