lean2/tests/lean/tactic3.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

12 lines
342 B
Text

Set: pp::colors
Set: pp::unicode
Assumed: p
Assumed: q
Assumed: r
Proved: T1
theorem T1 : p ⇒ p ∧ q ⇒ r ⇒ q ∧ r ∧ p :=
discharge
(λ H : p,
discharge
(λ H::1 : p ∧ q,
discharge (λ H::2 : r, and::intro (and::elimr H::1) (and::intro H::2 (and::eliml H::1)))))