Skip to content

Commit

Permalink
feat: add missing instance StarAlgEquivClass.toAlgEquivClass (#5160)
Browse files Browse the repository at this point in the history
  • Loading branch information
j-loreaux committed Jun 20, 2023
1 parent e266a22 commit 944d568
Showing 1 changed file with 11 additions and 1 deletion.
12 changes: 11 additions & 1 deletion Mathlib/Algebra/Star/StarAlgHom.lean
Expand Up @@ -8,9 +8,10 @@ Authors: Jireh Loreaux
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
import Mathlib.Algebra.Algebra.Equiv
import Mathlib.Algebra.Algebra.Prod
import Mathlib.Algebra.Hom.NonUnitalAlg
import Mathlib.Algebra.Star.Prod
import Mathlib.Algebra.Algebra.Prod

/-!
# Morphisms of star algebras
Expand Down Expand Up @@ -743,6 +744,15 @@ instance (priority := 100) (F R A B : Type _) [CommSemiring R] [Semiring A]
map_zero := map_zero
commutes := fun f r => by simp only [Algebra.algebraMap_eq_smul_one, map_smul, map_one] }

-- See note [lower instance priority]
instance (priority := 100) toAlgEquivClass {F R A B : Type _} [CommSemiring R]
[Ring A] [Ring B] [Algebra R A] [Algebra R B] [Star A] [Star B] [StarAlgEquivClass F R A B] :
AlgEquivClass F R A B :=
{ StarAlgEquivClass.toRingEquivClass,
StarAlgEquivClass.instStarAlgHomClass F R A B with
coe := fun f => f
inv := fun f => EquivLike.inv f }

end StarAlgEquivClass

namespace StarAlgEquiv
Expand Down

0 comments on commit 944d568

Please sign in to comment.