lean2/tests/lean/tst17.lean.expected.out
Leonardo de Moura 048151487e feat(kernel): use Pi as forall/implication
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-08 00:38:39 -08:00

7 lines
219 B
Text

Set: pp::colors
Set: pp::unicode
Assumed: f
Assumed: g
∀ a b : Type, ∃ c : Type, g a b = f c
∀ a b : Type, ∃ c : Type, g a b = f c : Bool
∀ (a b : Type), (∀ (x : Type), g a b == f x → ⊥) → ⊥