Skip to content

Commit

Permalink
feat(data/equiv): symm_symm_apply (#5324)
Browse files Browse the repository at this point in the history
A little dsimp lemma that's often helpful

Co-authored-by: Bryan Gin-ge Chen <bryangingechen@gmail.com>
  • Loading branch information
b-mehta and bryangingechen committed Dec 11, 2020
1 parent 63e1ad4 commit 846ee3f
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/data/equiv/basic.lean
Expand Up @@ -187,6 +187,10 @@ e.left_inv x
@[simp] lemma symm_trans_apply (f : α ≃ β) (g : β ≃ γ) (a : γ) :
(f.trans g).symm a = f.symm (g.symm a) := rfl

-- The `simp` attribute is needed to make this a `dsimp` lemma.
-- `simp` will always rewrite with `equiv.symm_symm` before this has a chance to fire.
@[simp, nolint simp_nf] theorem symm_symm_apply (f : α ≃ β) (b : α) : f.symm.symm b = f b := rfl

@[simp] theorem apply_eq_iff_eq (f : α ≃ β) {x y : α} : f x = f y ↔ x = y :=
f.injective.eq_iff

Expand Down

0 comments on commit 846ee3f

Please sign in to comment.