Linearly disjoint subalgebras #
This file contains basics about linearly disjoint subalgebras.
We adapt the definitions in https://en.wikipedia.org/wiki/Linearly_disjoint.
See the file Mathlib/LinearAlgebra/LinearDisjoint.lean for details.
Main definitions #
- Subalgebra.LinearDisjoint: two subalgebras are linearly disjoint, if they are linearly disjoint as submodules (- Submodule.LinearDisjoint).
- Subalgebra.LinearDisjoint.mulMap: if two subalgebras- Aand- Bof- S / Rare linearly disjoint, then there is- A ⊗[R] B ≃ₐ[R] A ⊔ Binduced by multiplication in- S.
Main results #
Equivalent characterization of linear disjointness #
- Subalgebra.LinearDisjoint.linearIndependent_left_of_flat: if- Aand- Bare linearly disjoint, and if- Bis a flat- R-module, then for any family of- R-linearly independent elements of- A, they are also- B-linearly independent.
- Subalgebra.LinearDisjoint.of_basis_left_op: conversely, if a basis of- Ais also- B-linearly independent, then- Aand- Bare linearly disjoint.
- Subalgebra.LinearDisjoint.linearIndependent_right_of_flat: if- Aand- Bare linearly disjoint, and if- Ais a flat- R-module, then for any family of- R-linearly independent elements of- B, they are also- A-linearly independent.
- Subalgebra.LinearDisjoint.of_basis_right: conversely, if a basis of- Bis also- A-linearly independent, then- Aand- Bare linearly disjoint.
- Subalgebra.LinearDisjoint.linearIndependent_mul_of_flat: if- Aand- Bare linearly disjoint, and if one of- Aand- Bis flat, then for any family of- R-linearly independent elements- { a_i }of- A, and any family of- R-linearly independent elements- { b_j }of- B, the family- { a_i * b_j }in- Sis also- R-linearly independent.
- Subalgebra.LinearDisjoint.of_basis_mul: conversely, if- { a_i }is an- R-basis of- A, if- { b_j }is an- R-basis of- B, such that the family- { a_i * b_j }in- Sis- R-linearly independent, then- Aand- Bare linearly disjoint.
Equivalent characterization by IsDomain or IsField of tensor product #
The following results are related to the equivalent characterizations in https://mathoverflow.net/questions/8324.
- Subalgebra.LinearDisjoint.isDomain_of_injective,- Subalgebra.LinearDisjoint.exists_field_of_isDomain_of_injective: under some flatness and injectivity conditions, if- Aand- Bare- R-algebras, then- A ⊗[R] Bis a domain if and only if there exists an- R-algebra which is a field that- Aand- Bembed into with linearly disjoint images.
- Subalgebra.LinearDisjoint.of_isField,- Subalgebra.LinearDisjoint.of_isField': if- A ⊗[R] Bis a field, then- Aand- Bare linearly disjoint, moreover, for any- R-algebra- Sand injections of- Aand- Binto- S, their images are linearly disjoint.
- Algebra.TensorProduct.not_isField_of_transcendental,- Algebra.TensorProduct.isAlgebraic_of_isField: if- Aand- Bare flat- R-algebras, both of them are transcendental, then- A ⊗[R] Bcannot be a field, equivalently, if- A ⊗[R] Bis a field, then one of them is algebraic.
Other main results #
- Subalgebra.LinearDisjoint.symm_of_commute,- Subalgebra.linearDisjoint_comm_of_commute: linear disjointness is symmetric under some commutative conditions.
- Subalgebra.LinearDisjoint.map: linear disjointness is preserved by injective algebra homomorphisms.
- Subalgebra.LinearDisjoint.bot_left,- Subalgebra.LinearDisjoint.bot_right: the image of- Rin- Sis linearly disjoint with any other subalgebras.
- Subalgebra.LinearDisjoint.sup_free_of_free: the compositum of two linearly disjoint subalgebras is a free module, if two subalgebras are also free modules.
- Subalgebra.LinearDisjoint.rank_sup_of_free,- Subalgebra.LinearDisjoint.finrank_sup_of_free: if subalgebras- Aand- Bare linearly disjoint and they are free modules, then the rank of- A ⊔ Bis equal to the product of the rank of- Aand- B.
- Subalgebra.LinearDisjoint.of_finrank_sup_of_free: conversely, if- Aand- Bare subalgebras which are free modules of finite rank, such that rank of- A ⊔ Bis equal to the product of the rank of- Aand- B, then- Aand- Bare linearly disjoint.
- Subalgebra.LinearDisjoint.adjoin_rank_eq_rank_left:- Subalgebra.LinearDisjoint.adjoin_rank_eq_rank_right: if- Aand- Bare linearly disjoint, if- Ais free and- Bis flat (resp.- Bis free and- Ais flat), then- [B[A] : B] = [A : R](resp.- [A[B] : A] = [B : R]). See also- Subalgebra.adjoin_rank_le.
- Subalgebra.LinearDisjoint.of_finrank_coprime_of_free: if the rank of- Aand- Bare coprime, and they satisfy some freeness condition, then- Aand- Bare linearly disjoint.
- Subalgebra.LinearDisjoint.inf_eq_bot_of_commute,- Subalgebra.LinearDisjoint.inf_eq_bot: if- Aand- Bare linearly disjoint, under suitable technical conditions, they are disjoint.
The results with name containing "of_commute" also have corresponding specialized versions
assuming S is commutative.
Tags #
linearly disjoint, linearly independent, tensor product
If A and B are subalgebras of S / R,
then A and B are linearly disjoint, if they are linearly disjoint as submodules of S.
Equations
Instances For
Linear disjointness is symmetric if elements in the module commute.
Linear disjointness is symmetric if elements in the module commute.
Linear disjointness is preserved by injective algebra homomorphisms.
The image of R in S is linearly disjoint with any other subalgebras.
The image of R in S is linearly disjoint with any other subalgebras.
Images of two R-algebras A and B in A ⊗[R] B are linearly disjoint.
Linear disjointness is symmetric in a commutative ring.
Linear disjointness is symmetric in a commutative ring.
Two subalgebras A, B in a commutative ring are linearly disjoint if and only if
Subalgebra.mulMap A B is injective.
If A and B are subalgebras in a commutative algebra S over R, and if they are
linearly disjoint, then there is the natural isomorphism
A ⊗[R] B ≃ₐ[R] A ⊔ B induced by multiplication in S.
Equations
Instances For
If A and B are linearly disjoint subalgebras in a commutative algebra S over R
such that A ⊔ B = S, then this is the natural isomorphism
A ⊗[R] B ≃ₐ[A] S induced by multiplication in S.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If A and B are linearly disjoint subalgebras in a commutative algebra S over R
such that A ⊔ B = S, then any R-basis of B is also an A-basis of S.
Equations
- H.basisOfBasisRight H' b = (Module.Basis.baseChange (↥A) b).map (H.mulMapLeftOfSupEqTop H').toLinearEquiv
Instances For
If A and B are subalgebras in a commutative algebra S over R, and if they are
linearly disjoint and such that A ⊔ B = S, then any R-basis of A is also a B-basis of S.
Equations
- H.basisOfBasisLeft H' b = (Module.Basis.baseChange (↥B) b).map (⋯.mulMapLeftOfSupEqTop ⋯).toLinearEquiv
Instances For
If A and B are subalgebras in a commutative algebra S over R, and if they are
linearly disjoint, and if they are free R-modules, then A ⊔ B is also a free R-module.
If A and B are subalgebras in a domain S over R, and if they are
linearly disjoint, then A ⊗[R] B is also a domain.
If A and B are R-algebras, such that there exists a domain S over R
such that A and B inject into it and their images are linearly disjoint,
then A ⊗[R] B is also a domain.
If A and B are linearly disjoint, if B is a flat R-module, then for any family of
R-linearly independent elements of A, they are also B-linearly independent
in the opposite ring.
If a basis of A is also B-linearly independent in the opposite ring,
then A and B are linearly disjoint.
If A and B are linearly disjoint, if A is a flat R-module, then for any family of
R-linearly independent elements of B, they are also A-linearly independent.
If a basis of B is also A-linearly independent, then A and B are linearly disjoint.
If A and B are linearly disjoint and their elements commute, if B is a flat R-module,
then for any family of R-linearly independent elements of A,
they are also B-linearly independent.
If a basis of A is also B-linearly independent, if elements in A and B commute,
then A and B are linearly disjoint.
If A and B are linearly disjoint, if A is flat, then for any family of
R-linearly independent elements { a_i } of A, and any family of
R-linearly independent elements { b_j } of B, the family { a_i * b_j } in S is
also R-linearly independent.
If A and B are linearly disjoint, if B is flat, then for any family of
R-linearly independent elements { a_i } of A, and any family of
R-linearly independent elements { b_j } of B, the family { a_i * b_j } in S is
also R-linearly independent.
If A and B are linearly disjoint, if one of A and B is flat, then for any family of
R-linearly independent elements { a_i } of A, and any family of
R-linearly independent elements { b_j } of B, the family { a_i * b_j } in S is
also R-linearly independent.
If { a_i } is an R-basis of A, if { b_j } is an R-basis of B,
such that the family { a_i * b_j } in S is R-linearly independent,
then A and B are linearly disjoint.
If A and B are subalgebras in a commutative algebra S over R, and if they are
linearly disjoint and such that A ⊔ B = S, then trace and algebraMap commutes.
If A and B are subalgebras in a commutative algebra S over R, and if they are
linearly disjoint and such that A ⊔ B = S, then norm and algebraMap commutes.
In a commutative ring, if A and B are linearly disjoint, if B is a flat R-module,
then for any family of R-linearly independent elements of A,
they are also B-linearly independent.
In a commutative ring, if a basis of A is also B-linearly independent,
then A and B are linearly disjoint.
If A and B are flat algebras over R, such that A ⊗[R] B is a domain, and such that
the algebra maps are injective, then there exists an R-algebra K that is a field that A
and B inject into with linearly disjoint images. Note: K can chosen to be the
fraction field of A ⊗[R] B, but here we hide this fact.
If A ⊗[R] B is a field, then A and B are linearly disjoint.
If A ⊗[R] B is a field, then for any R-algebra S
and injections of A and B into S, their images are linearly disjoint.
If A and B are flat R-algebras, both of them are transcendental, then A ⊗[R] B cannot
be a field.
If A and B are flat R-algebras, such that A ⊗[R] B is a field, then one of A and B
is algebraic over R.
In a commutative ring, if subalgebras A and B are linearly disjoint and they are
free modules, then the rank of A ⊔ B is equal to the product of the rank of A and B.
In a commutative ring, if subalgebras A and B are linearly disjoint and they are
free modules, then the rank of A ⊔ B is equal to the product of the rank of A and B.
In a commutative ring, if A and B are subalgebras which are free modules of finite rank,
such that rank of A ⊔ B is equal to the product of the rank of A and B,
then A and B are linearly disjoint.
If A and B are linearly disjoint, if A is free and B is flat,
then [B[A] : B] = [A : R]. See also Subalgebra.adjoin_rank_le.
If A and B are linearly disjoint, if B is free and A is flat,
then [A[B] : A] = [B : R]. See also Subalgebra.adjoin_rank_le.
If the rank of A and B are coprime, and they satisfy some freeness condition,
then A and B are linearly disjoint.
If A/R is integral, such that A' and B are linearly disjoint for all subalgebras A'
of A which are finitely generated R-modules, then A and B are linearly disjoint.
If B/R is integral, such that A and B' are linearly disjoint for all subalgebras B'
of B which are finitely generated R-modules, then A and B are linearly disjoint.
If A/R and B/R are integral, such that any finite subalgebras in A and B are
linearly disjoint, then A and B are linearly disjoint.