lean2/tests/lean/tactic1.lean.expected.out

7 lines
177 B
Text
Raw Normal View History

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