lean2/tests/lean/disj1.lean.expected.out

7 lines
200 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Proved: T1
Proved: T2
Theorem T2 (a b : Bool) : a b ⇒ b a :=
Discharge (λ H : a b, DisjCases H (λ H : a, Disj2 b H) (λ H : b, Disj1 a H))