Tensor product and products #
In this file we examine the behaviour of the tensor product with arbitrary and finite products.
Let S
be an R
-algebra, N
an S
-module, ι
an index type and Mᵢ
a family of R
-modules.
We then have a natural map
TensorProduct.piRightHom
: N ⊗[R] (∀ i, M i) →ₗ[S] ∀ i, N ⊗[R] M i
In general, this is not an isomorphism, but if ι
is finite, then it is
and it is packaged as TensorProduct.piRight
. Also a special case for when Mᵢ = R
is given.
Notes #
See Mathlib.LinearAlgebra.TensorProduct.Prod
for binary products.
For any R
-module N
, index type ι
and family of R
-modules Mᵢ
, there is a natural
linear map N ⊗[R] (∀ i, M i) →ₗ ∀ i, N ⊗[R] M i
. This map is an isomorphism if ι
is finite.
Equations
Instances For
Tensor product commutes with finite products on the right.
Equations
- TensorProduct.piRight R S N M = LinearEquiv.ofLinear (TensorProduct.piRightHom R S N M) (TensorProduct.piRightInv R S N M) ⋯ ⋯
Instances For
For any R
-module N
and index type ι
, there is a natural
linear map N ⊗[R] (ι → R) →ₗ (ι → N)
. This map is an isomorphism if ι
is finite.
Equations
Instances For
For any R
-module N
and finite index type ι
, N ⊗[R] (ι → R)
is canonically
isomorphic to ι → N
.
Equations
- TensorProduct.piScalarRight R S N ι = LinearEquiv.ofLinear (TensorProduct.piScalarRightHom R S N ι) (TensorProduct.piScalarRightInv R S N ι) ⋯ ⋯