lean2/tests/lean/tst16.lean.expected.out

16 lines
590 B
Text
Raw Normal View History

Assumed: f
∀ a b : Type, (f a) = (f b)
Assumed: g
∀ (a b : Type) (c : Bool), g c ((f a) = (f b))
∃ (a b : Type) (c : Bool), g c ((f a) = (f b))
∀ (a b : Type) (c : Bool), (g c (f a)) = (f b) ⇒ (f a)
Bool
∀ (a b : Type) (c : Bool), g c ((f a) = (f b))
∀ a b : Type, (f a) = (f b)
∃ a b : Type, (f a) = (f b) ∧ (f a)
∃ a b : Type, (f a) = (f b) (f b)
Assumed: a
(f a) (f a)
(f a) = a (f a)
(f a) = a ∧ (f a)