lean2/tests/lean/run/apply_failure.lean

6 lines
146 B
Text
Raw Normal View History

example (a b c : Prop) : a ∧ b → b ∧ a :=
begin
intro H,
repeat (apply or.elim H | apply and.elim H | intro H | split | assumption)
end