Skip to content

Commit

Permalink
rm Module.endUnitsToModuleAutEquiv
Browse files Browse the repository at this point in the history
  • Loading branch information
ScottCarnahan committed Oct 30, 2024
1 parent e8d24de commit 2f2440b
Showing 1 changed file with 0 additions and 13 deletions.
13 changes: 0 additions & 13 deletions Mathlib/Algebra/Module/Equiv/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -196,19 +196,6 @@ def toModuleAut : S →* M ≃ₗ[R] M where

end DistribMulAction

/-- An isomorphism from invertible linear endomorphisms to linear automorphisms. -/
def Module.endUnitsToModuleAutEquiv (R) (M) [CommRing R] [AddCommGroup M] [Module R M] :
(M →ₗ[R] M)ˣ ≃* (M ≃ₗ[R] M) where
toFun f := DistribMulAction.toLinearEquiv R M f
invFun f := ⟨f, f.symm, by ext; simp, by ext; simp⟩
left_inv f := by ext; simp [Units.smul_def]
right_inv f := by ext; simp
map_mul' f g := by
ext x
simp only [DistribMulAction.toLinearEquiv_apply, mul_smul,
show (DistribMulAction.toLinearEquiv R M f * DistribMulAction.toLinearEquiv R M g) x =
DistribMulAction.toLinearEquiv R M f ((DistribMulAction.toLinearEquiv R M g) x) by rfl]

namespace AddEquiv

section AddCommMonoid
Expand Down

0 comments on commit 2f2440b

Please sign in to comment.