lean2/tests/lean/tst10.lean.expected.out
Leonardo de Moura 51640ecff8 Move files in examples directory to tests directory. They are not real examples
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-08-31 19:16:30 -07:00

255 B
Raw Blame History

Assumed: a
Assumed: b
a ∧ b
a ∧ b ∧ a
a ∧ b
a ∧ b
a ∧ b
a ∧ b
a b
a b
a b
a b
a a b
a ⇒ b ⇒ a
Bool
ite Bool a a
a
Assumed: H1
Assumed: H2
Π (a b : Bool) (H1 : a ⇒ b) (H2 : a), b
MP H2 H1
b