lean2/tests/lean/run/match_tac2.lean
Leonardo de Moura e379034b95 feat(library/tactic): improve 'assumption' tactic
- It uses the unifier in "conservative" mode
- It only affects the current goal

closes #570
2015-05-02 17:33:54 -07:00

12 lines
284 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; repeat assumption
end},
{intro H,
match H with
| and.intro H₁ H₂ := by apply and.intro; repeat assumption
end},
end