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

18 lines
534 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
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)
∀ (a b : Type) (c : Bool), g c ((f a) = (f b)) : 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)