lean2/tests/lean/tactic8.lean.expected.out

6 lines
219 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Proved: T
theorem T (a b : Bool) : a b ⇒ ¬ b ⇒ a :=
discharge (λ H : a b, discharge (λ H::1 : ¬ b, or::elim H (λ H : a, H) (λ H : b, absurd::elim a H H::1)))