Interaction between Quotients and Tensor Products #
This file contains constructions that relate quotients and tensor products.
Let M, N
be R
-modules, m ≤ M
and n ≤ N
be an R
-submodules and I ≤ R
an ideal. We prove
the following isomorphisms:
Main results #
TensorProduct.quotientTensorQuotientEquiv
:(M ⧸ m) ⊗[R] (N ⧸ n) ≃ₗ[R] (M ⊗[R] N) ⧸ (m ⊗ N ⊔ M ⊗ n)
TensorProduct.quotientTensorEquiv
:(M ⧸ m) ⊗[R] N ≃ₗ[R] (M ⊗[R] N) ⧸ (m ⊗ N)
TensorProduct.tensorQuotientEquiv
:M ⊗[R] (N ⧸ n) ≃ₗ[R] (M ⊗[R] N) ⧸ (M ⊗ n)
TensorProduct.quotTensorEquivQuotSMul
:(R ⧸ I) ⊗[R] M ≃ₗ[R] M ⧸ (I • M)
TensorProduct.tensorQuotEquivQuotSMul
:M ⊗[R] (R ⧸ I) ≃ₗ[R] M ⧸ (I • M)
Tags #
Quotient, Tensor Product
Let M, N
be R
-modules, m ≤ M
and n ≤ N
be an R
-submodules. Then we have a linear
isomorphism between tensor products of the quotients and the quotient of the tensor product:
(M ⧸ m) ⊗[R] (N ⧸ n) ≃ₗ[R] (M ⊗[R] N) ⧸ (m ⊗ N ⊔ M ⊗ n)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Let M, N
be R
-modules, m ≤ M
be an R
-submodule. Then we have a linear isomorphism between
tensor products of the quotient and the quotient of the tensor product:
(M ⧸ m) ⊗[R] N ≃ₗ[R] (M ⊗[R] N) ⧸ (m ⊗ N)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Let M, N
be R
-modules, n ≤ N
be an R
-submodule. Then we have a linear isomorphism between
tensor products of the quotient and the quotient of the tensor product:
M ⊗[R] (N ⧸ n) ≃ₗ[R] (M ⊗[R] N) ⧸ (M ⊗ n)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Left tensoring a module with a quotient of the ring is the same as quotienting that module by the corresponding submodule.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Right tensoring a module with a quotient of the ring is the same as quotienting that module by the corresponding submodule.
Equations
- TensorProduct.tensorQuotEquivQuotSMul M I = (TensorProduct.comm R M (R ⧸ I)).trans (TensorProduct.quotTensorEquivQuotSMul M I)