Maps between tensor products of R-algebras #
This file provides results about maps between tensor products of R-algebras.
Main declarations #
- the structure isomorphisms
Algebra.TensorProduct.lid : R ⊗[R] A ≃ₐ[R] AAlgebra.TensorProduct.rid : A ⊗[R] R ≃ₐ[S] A(usually used withS = RorS = A)Algebra.TensorProduct.comm : A ⊗[R] B ≃ₐ[R] B ⊗[R] AAlgebra.TensorProduct.assoc : ((A ⊗[R] B) ⊗[R] C) ≃ₐ[R] (A ⊗[R] (B ⊗[R] C))
Algebra.TensorProduct.liftEquiv: a universal property for the tensor product of algebras.
References #
The map LinearMap.lTensorHom which sends f ↦ 1 ⊗ f as a morphism of algebras.
Equations
- Module.End.lTensorAlgHom R M N = AlgHom.ofLinearMap (LinearMap.lTensorHom N) ⋯ ⋯
Instances For
The map LinearMap.rTensorHom which sends f ↦ f ⊗ 1 as a morphism of algebras.
Equations
- Module.End.rTensorAlgHom R M N = AlgHom.ofLinearMap (LinearMap.rTensorHom N) ⋯ ⋯
Instances For
We build the structure maps for the symmetric monoidal category of R-algebras.
To check a linear map preserves multiplication, it suffices to check it on pure tensors. See
algHomOfLinearMapTensorProduct for a bundled version.
Build an algebra morphism from a linear map out of a tensor product, and evidence that on pure tensors, it preserves multiplication and the identity.
Note that we state h_one using 1 ⊗ₜ[R] 1 instead of 1 so that lemmas about f applied to pure
tensors can be directly applied by the caller (without needing TensorProduct.one_def).
Equations
- Algebra.TensorProduct.algHomOfLinearMapTensorProduct f h_mul h_one = AlgHom.ofLinearMap f h_one ⋯
Instances For
Build an algebra equivalence from a linear equivalence out of a tensor product, and evidence that on pure tensors, it preserves multiplication and the identity.
Note that we state h_one using 1 ⊗ₜ[R] 1 instead of 1 so that lemmas about f applied to pure
tensors can be directly applied by the caller (without needing TensorProduct.one_def).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Build an algebra equivalence from a linear equivalence out of a triple tensor product, and evidence of multiplicativity on pure tensors.
Equations
- Algebra.TensorProduct.algEquivOfLinearEquivTripleTensorProduct f h_mul h_one = AlgEquiv.ofLinearEquiv f h_one ⋯
Instances For
The forward direction of the universal property of tensor products of algebras; any algebra morphism from the tensor product can be factored as the product of two algebra morphisms that commute.
See Algebra.TensorProduct.liftEquiv for the fact that every morphism factors this way.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The universal property of the tensor product of algebras.
Pairs of algebra morphisms that commute are equivalent to algebra morphisms from the tensor product.
This is Algebra.TensorProduct.lift as an equivalence.
See also GradedTensorProduct.liftEquiv for an alternative commutativity requirement for graded
algebra.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The base ring is a left identity for the tensor product of algebra, up to algebra isomorphism.
Equations
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.
Equations
Instances For
If A and B are both R- and S-algebras and their actions on them commute,
and if the S-action on A ⊗[R] B can switch between the two factors, then there is a
canonical S-algebra homomorphism from A ⊗[S] B to A ⊗[R] B.
Equations
- Algebra.TensorProduct.mapOfCompatibleSMul R S A B = AlgHom.ofLinearMap (TensorProduct.mapOfCompatibleSMul R S A B) ⋯ ⋯
Instances For
mapOfCompatibleSMul R S A B is also A-linear.
Equations
- Algebra.TensorProduct.mapOfCompatibleSMul' R S A B = AlgHom.ofLinearMap (TensorProduct.mapOfCompatibleSMul' R S A B) ⋯ ⋯
Instances For
If the R- and S-actions on A and B satisfy CompatibleSMul both ways,
then A ⊗[S] B is canonically isomorphic to A ⊗[R] B.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If the R- and S- action on S and A satisfy CompatibleSMul both ways,
then S ⊗[R] A is canonically isomorphic to A.
Equations
Instances For
The tensor product of R-algebras is commutative, up to algebra isomorphism.
Equations
Instances For
The associator for tensor product of R-algebras, as an algebra isomorphism.
Equations
- Algebra.TensorProduct.assoc R S A C D = AlgEquiv.ofLinearEquiv (TensorProduct.AlgebraTensorModule.assoc R S S A C D) ⋯ ⋯
Instances For
The natural isomorphism A ⊗[S] (S ⊗[R] B) ≃ₐ[T] A ⊗[R] B.
Equations
- Algebra.TensorProduct.cancelBaseChange R S T A B = (AlgEquiv.ofLinearEquiv (TensorProduct.AlgebraTensorModule.cancelBaseChange R S T A B).symm ⋯ ⋯).symm
Instances For
The tensor product of a pair of algebra morphisms.
Equations
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.
Equations
- Algebra.TensorProduct.congr f g = AlgEquiv.ofAlgHom (Algebra.TensorProduct.map ↑f ↑g) (Algebra.TensorProduct.map ↑f.symm ↑g.symm) ⋯ ⋯
Instances For
Tensor product of algebras analogue of mul_left_comm.
This is the algebra version of TensorProduct.leftComm.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Tensor product of algebras analogue of mul_mul_mul_comm.
This is the algebra version of TensorProduct.AlgebraTensorModule.tensorTensorTensorComm.
Equations
- Algebra.TensorProduct.tensorTensorTensorComm R R' S T A B C D = AlgEquiv.ofLinearEquiv (TensorProduct.AlgebraTensorModule.tensorTensorTensorComm R R' S T A B C D) ⋯ ⋯
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.
This is just a special case of Algebra.TensorProduct.lift for when C is commutative.
Equations
Instances For
LinearMap.mul' as an AlgHom over the algebra.
Equations
- Algebra.TensorProduct.lmul'' R = Algebra.TensorProduct.algHomOfLinearMapTensorProduct (let __spread.0 := LinearMap.mul' R S; { toAddHom := __spread.0.toAddHom, map_smul' := ⋯ }) ⋯ ⋯
Instances For
LinearMap.mul' as an AlgHom over the base ring.
Equations
Instances For
If multiplication by elements of S can switch between the two factors of S ⊗[R] S,
then lmul'' is an isomorphism.
Equations
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).
This is a special case of Algebra.TensorProduct.productLeftAlgHom for when the two base rings are
the same.
Equations
Instances For
The natural linear map $A ⊗ \text{Hom}_R(M, N) → \text{Hom}_A (M_A, N_A)$, where $M_A$ and $N_A$ are the respective modules over $A$ obtained by extension of scalars.
See LinearMap.tensorProductEnd for this map specialized to endomorphisms,
and bundled as A-algebra homomorphism.
Equations
- LinearMap.tensorProduct R A M N = TensorProduct.AlgebraTensorModule.lift { toFun := fun (a : A) => a • LinearMap.baseChangeHom R A M N, map_add' := ⋯, map_smul' := ⋯ }
Instances For
The natural A-algebra homomorphism $A ⊗ (\text{End}_R M) → \text{End}_A (A ⊗ M)$,
where M is an R-module, and A an R-algebra.
Equations
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.