Skip to content

Commit

Permalink
Add helper FunLike instance for AlgEquiv
Browse files Browse the repository at this point in the history
  • Loading branch information
Vierkantor committed Nov 27, 2023
1 parent 9b936db commit d167b2b
Showing 1 changed file with 5 additions and 0 deletions.
5 changes: 5 additions & 0 deletions Mathlib/Algebra/Algebra/Equiv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -109,6 +109,11 @@ instance : EquivLike (A₁ ≃ₐ[R] A₂) A₁ A₂ where
obtain ⟨⟨g,_⟩,_⟩ := g
congr

/-- Helper instance since the coercion is not always found. -/
instance : NDFunLike (A₁ ≃ₐ[R] A₂) A₁ A₂ where
coe := FunLike.coe
coe_injective' := FunLike.coe_injective'

instance : AlgEquivClass (A₁ ≃ₐ[R] A₂) R A₁ A₂ where
map_add f := f.map_add'
map_mul f := f.map_mul'
Expand Down

0 comments on commit d167b2b

Please sign in to comment.