lean2/tests/lean/tactic5.lean.expected.out
Leonardo de Moura 935c2a03a3 feat(*): change name conventions for Lean builtin libraries
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-05 19:21:44 -08:00

5 lines
189 B
Text

Set: pp::colors
Set: pp::unicode
Proved: T4
theorem T4 (a b : Bool) : a ⇒ b ⇒ a ∧ b ∧ a :=
discharge (λ H : a, discharge (λ H::1 : b, and::intro H (and::intro H::1 H)))