Skip to content

Commit

Permalink
delete duplicate
Browse files Browse the repository at this point in the history
  • Loading branch information
zjj committed Jan 31, 2025
1 parent 165390e commit 6492080
Showing 1 changed file with 0 additions and 5 deletions.
5 changes: 0 additions & 5 deletions Mathlib/Algebra/Category/ModuleCat/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -470,11 +470,6 @@ variable (M N : ModuleCat.{v} R)
/-- `ModuleCat.Hom.hom` as an isomorphism of monoids. -/
@[deprecated (since := "2025-01-23")] alias endMulEquiv := endRingEquiv

/-- `ModuleCat.Hom.hom` as an isomorphism of rings. -/
@[simps!] def endRingEquiv : End M ≃+* (M →ₗ[R] M) where
__ := endMulEquiv M
map_add' _ _ := rfl

/-- The scalar multiplication on an object of `ModuleCat R` considered as
a morphism of rings from `R` to the endomorphisms of the underlying abelian group. -/
def smul : R →+* End ((forget₂ (ModuleCat R) AddCommGrp).obj M) where
Expand Down

0 comments on commit 6492080

Please sign in to comment.