The tensor product of R-algebras #
This file provides results about the multiplicative structure on A ⊗[R] B
when R
is a
commutative (semi)ring and A
and B
are both R
-algebras. On these tensor products,
multiplication is characterized by (a₁ ⊗ₜ b₁) * (a₂ ⊗ₜ b₂) = (a₁ * a₂) ⊗ₜ (b₁ * b₂)
.
Main declarations #
LinearMap.baseChange A f
is theA
-linear mapA ⊗ f
, for anR
-linear mapf
.Algebra.TensorProduct.semiring
: the ring structure onA ⊗[R] B
for twoR
-algebrasA
,B
.Algebra.TensorProduct.leftAlgebra
: theS
-algebra structure onA ⊗[R] B
, for whenA
is additionally anS
algebra.- the structure isomorphisms
Algebra.TensorProduct.lid : R ⊗[R] A ≃ₐ[R] A
Algebra.TensorProduct.rid : A ⊗[R] R ≃ₐ[S] A
(usually used withS = R
orS = A
)Algebra.TensorProduct.comm : A ⊗[R] B ≃ₐ[R] B ⊗[R] A
Algebra.TensorProduct.assoc : ((A ⊗[R] B) ⊗[R] C) ≃ₐ[R] (A ⊗[R] (B ⊗[R] C))
The base-change of a linear map of R
-modules to a linear map of A
-modules #
baseChange A f
for f : M →ₗ[R] N
is the A
-linear map A ⊗[R] M →ₗ[A] A ⊗[R] N
.
Instances For
baseChange
as a linear map.
Instances For
The R
-algebra structure on A ⊗[R] B
#
(Implementation detail)
The multiplication map on A ⊗[R] B
,
for a fixed pure tensor in the first argument,
as an R
-linear map.
Instances For
(Implementation detail)
The multiplication map on A ⊗[R] B
,
as an R
-bilinear map.
Instances For
The ring morphism A →+* A ⊗[R] B
sending a
to a ⊗ₜ 1
.
Instances For
The tensor product of two R
-algebras is an R
-algebra.
The R
-algebra morphism A →ₐ[R] A ⊗[R] B
sending a
to a ⊗ₜ 1
.
Instances For
The algebra morphism B →ₐ[R] A ⊗[R] B
sending b
to 1 ⊗ₜ b
.
Instances For
A version of TensorProduct.ext
for AlgHom
.
Using this as the @[ext]
lemma instead of Algebra.TensorProduct.ext'
allows ext
to apply
lemmas specific to A →ₐ[S] _
and B →ₐ[R] _
; notably this allows recursion into nested tensor
products of algebras.
See note [partially-applied ext lemmas].
S ⊗[R] T
has a T
-algebra structure. This is not a global instance or else the action of
S
on S ⊗[R] S
would be ambiguous.
Instances For
We now build the structure maps for the symmetric monoidal category of R
-algebras.
Build an algebra morphism from a linear map out of a tensor product, and evidence of multiplicativity on pure tensors.
Instances For
Build an algebra equivalence from a linear equivalence out of a tensor product, and evidence of multiplicativity on pure tensors.
Instances For
Build an algebra equivalence from a linear equivalence out of a triple tensor product, and evidence of multiplicativity on pure tensors.
Instances For
The base ring is a left identity for the tensor product of algebra, up to algebra isomorphism.
Instances For
The base ring is a right identity for the tensor product of algebra, up to algebra isomorphism.
Note that if A
is commutative this can be instantiated with S = A
.
Instances For
The tensor product of R-algebras is commutative, up to algebra isomorphism.
Instances For
The associator for tensor product of R-algebras, as an algebra isomorphism.
Instances For
The tensor product of a pair of algebra morphisms.
Instances For
Construct an isomorphism between tensor products of an S-algebra with an R-algebra from S- and R- isomorphisms between the tensor factors.
Instances For
LinearMap.mul'
is an AlgHom
on commutative rings.
Instances For
If S
is commutative, for a pair of morphisms f : A →ₐ[R] S
, g : B →ₐ[R] S
,
We obtain a map A ⊗[R] B →ₐ[R] S
that commutes with f
, g
via a ⊗ b ↦ f(a) * g(b)
.
Instances For
If A
, B
, C
are R
-algebras, A
and C
are also S
-algebras (forming a tower as
·/S/R
), then the product map of f : A →ₐ[S] C
and g : B →ₐ[R] C
is an S
-algebra
homomorphism.
Instances For
Given an R
-algebra A
and an R
-basis of M
, this is an R
-linear isomorphism
A ⊗[R] M ≃ (ι →₀ A)
(which is in fact A
-linear).
Instances For
Given a R
-algebra A
, this is the A
-basis of A ⊗[R] M
induced by a R
-basis of M
.
Instances For
The algebra homomorphism from End M ⊗ End N
to End (M ⊗ N)
sending f ⊗ₜ g
to
the TensorProduct.map f g
, the tensor product of the two maps.
This is an AlgHom
version of TensorProduct.AlgebraTensorModule.homTensorHomMap
. Like that
definition, this is generalized across many different rings; namely a tower of algebras A/S/R
.
Instances For
An auxiliary definition, used for constructing the Module (A ⊗[R] B) M
in
TensorProduct.Algebra.module
below.
Instances For
If M
is a representation of two different R
-algebras A
and B
whose actions commute,
then it is a representation the R
-algebra A ⊗[R] B
.
An important example arises from a semiring S
; allowing S
to act on itself via left and right
multiplication, the roles of R
, A
, B
, M
are played by ℕ
, S
, Sᵐᵒᵖ
, S
. This example
is important because a submodule of S
as a Module
over S ⊗[ℕ] Sᵐᵒᵖ
is a two-sided ideal.
NB: This is not an instance because in the case B = A
and M = A ⊗[R] A
we would have a diamond
of smul
actions. Furthermore, this would not be a mere definitional diamond but a true
mathematical diamond in which A ⊗[R] A
had two distinct scalar actions on itself: one from its
multiplication, and one from this would-be instance. Arguably we could live with this but in any
case the real fix is to address the ambiguity in notation, probably along the lines outlined here:
https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.234773.20base.20change/near/240929258