lean2/tests/lean/run/match_tac2.lean

12 lines
270 B
Text

example (a b c : Prop) : a ∧ b ↔ b ∧ a :=
begin
apply iff.intro,
{intro H,
match H with
| and.intro H₁ H₂ := by apply and.intro; assumption
end},
{intro H,
match H with
| and.intro H₁ H₂ := by apply and.intro; assumption
end},
end