lean2/tests/lean/tactic10.lean.expected.out

11 lines
281 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Defined: f
Defined: g
Proved: T1
Defined: h
Proved: T2
Theorem T2 (a b : Bool) : h a b ⇒ f b ⇒ a :=
Discharge
(λ H : a b, Discharge (λ H::1 : ¬ b, DisjCases H (λ H : a, H) (λ H : b, AbsurdImpAny b a H H::1)))