Skip to content

Commit

Permalink
Update Mathlib/Algebra/Azumaya/Defs.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Eric Wieser <[email protected]>
  • Loading branch information
Whysoserioushah and eric-wieser authored Jan 22, 2025
1 parent 0d72d72 commit de74508
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Azumaya/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -38,7 +38,7 @@ noncomputable abbrev instModuleTensorProductMop :
/-- The canonical map from `A ⊗[R] Aᵐᵒᵖ` to `Module.End R A` where
`a ⊗ b` maps to `f : x ↦ a * x * b`. -/
noncomputable abbrev AlgHom.tensorMopToEnd : (A ⊗[R] Aᵐᵒᵖ) →ₐ[R] Module.End R A :=
letI := instModuleTensorProductMop R A
letI : Module (A ⊗[R] Aᵐᵒᵖ) A := TensorProduct.Algebra.module
letI : IsScalarTower R (A ⊗[R] Aᵐᵒᵖ) A := {
smul_assoc := fun r ab a ↦ by
change TensorProduct.Algebra.moduleAux _ _ = _ • TensorProduct.Algebra.moduleAux _ _
Expand Down

0 comments on commit de74508

Please sign in to comment.