lean2/tests/lean/tactic9.lean.expected.out

7 lines
235 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Defined: f
Proved: T
Theorem T (a b : Bool) : a b ⇒ (f b) ⇒ a :=
Discharge (λ H : a b, Discharge (λ H::1 : f b, DisjCases H (λ H : a, H) (λ H : b, AbsurdImpAny b a H H::1)))