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

6 lines
176 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Defined: f
Proved: T
theorem T (a b : Bool) (H : a b) (H::1 : f b) : a := or_elim H (λ H : a, H) (λ H : b, absurd_elim a H H::1)