mathlib documentation

algebra.​category.​Module.​monoidal

algebra.​category.​Module.​monoidal

The monoidal category structure on R-modules

Mostly this uses existing machinery in linear_algebra.tensor_product. We just need to provide a few small missing pieces to build the monoidal_category instance.

If you're happy using the bundled Module R, it may be possible to mostly use this as an interface and not need to interact much with the implementation details.

(implementation) tensor product of R-modules

Equations

(implementation) tensor product of morphisms R-modules

Equations
theorem Module.​monoidal_category.​tensor_comp {R : Type u} [comm_ring R] {X₁ Y₁ Z₁ X₂ Y₂ Z₂ : Module R} (f₁ : X₁ Y₁) (f₂ : X₂ Y₂) (g₁ : Y₁ Z₁) (g₂ : Y₂ Z₂) :

theorem Module.​monoidal_category.​associator_naturality {R : Type u} [comm_ring R] {X₁ X₂ X₃ Y₁ Y₂ Y₃ : Module R} (f₁ : X₁ Y₁) (f₂ : X₂ Y₂) (f₃ : X₃ Y₃) :

(implementation) the left unitor for R-modules

Equations

(implementation) the right unitor for R-modules

Equations
@[instance]
def Module.​comm_ring {R : Type u} [comm_ring R] :

Remind ourselves that the monoidal unit, being just R, is still a commutative ring.

Equations
@[simp]
theorem Module.​monoidal_category.​left_unitor_hom {R : Type u} [comm_ring R] {M : Module R} (r : R) (m : M) :
((λ_ M).hom) (r ⊗ₜ[R] m) = r m

@[simp]
theorem Module.​monoidal_category.​right_unitor_hom {R : Type u} [comm_ring R] {M : Module R} (m : M) (r : R) :
((ρ_ M).hom) (m ⊗ₜ[R] r) = r m

@[simp]
theorem Module.​monoidal_category.​associator_hom {R : Type u} [comm_ring R] {M N K : Module R} (m : M) (n : N) (k : K) :
((α_ M N K).hom) ((m ⊗ₜ[R] n) ⊗ₜ[R] k) = m ⊗ₜ[R] n ⊗ₜ[R] k