Linearly disjoint fields #
This file contains basics about the linearly disjoint fields.
We adapt the definitions in https://en.wikipedia.org/wiki/Linearly_disjoint.
See the file Mathlib/LinearAlgebra/LinearDisjoint.lean
and Mathlib/RingTheory/LinearDisjoint.lean
for details.
Main definitions #
IntermediateField.LinearDisjoint
: an intermediate fieldA
ofE / F
and an abstract fieldL
betweenE / F
(as a special case, two intermediate fields) are linearly disjoint overF
, if they are linearly disjoint as subalgebras (Subalgebra.LinearDisjoint
).
Implementation notes #
The Subalgebra.LinearDisjoint
is stated for two Subalgebra
s. The original design of
IntermediateField.LinearDisjoint
is also stated for two IntermediateField
s
(see IntermediateField.linearDisjoint_iff'
for the original statement).
But it's probably useful if one of them can be generalized to an abstract field
(see https://github.com/leanprover-community/mathlib4/pull/9651#discussion_r1464070324).
This leads to the current design of IntermediateField.LinearDisjoint
which is for one IntermediateField
and one abstract field.
It is not generalized to two abstract fields as this will break the dot notation.
Main results #
Equivalent characterization of linear disjointness #
IntermediateField.LinearDisjoint.linearIndependent_left
: ifA
andL
are linearly disjoint, then anyF
-linearly independent family onA
remains linearly independent overL
.IntermediateField.LinearDisjoint.of_basis_left
: conversely, if there exists anF
-basis ofA
which remains linearly independent overL
, thenA
andL
are linearly disjoint.IntermediateField.LinearDisjoint.linearIndependent_right
:IntermediateField.LinearDisjoint.linearIndependent_right'
: ifA
andL
are linearly disjoint, then anyF
-linearly independent family onL
remains linearly independent overA
.IntermediateField.LinearDisjoint.of_basis_right
:IntermediateField.LinearDisjoint.of_basis_right'
: conversely, if there exists anF
-basis ofL
which remains linearly independent overA
, thenA
andL
are linearly disjoint.IntermediateField.LinearDisjoint.linearIndependent_mul
:IntermediateField.LinearDisjoint.linearIndependent_mul'
: ifA
andL
are linearly disjoint, then for any family ofF
-linearly independent elements{ a_i }
ofA
, and any family ofF
-linearly independent elements{ b_j }
ofL
, the family{ a_i * b_j }
inS
is alsoF
-linearly independent.IntermediateField.LinearDisjoint.of_basis_mul
:IntermediateField.LinearDisjoint.of_basis_mul'
: conversely, if{ a_i }
is anF
-basis ofA
, if{ b_j }
is anF
-basis ofL
, such that the family{ a_i * b_j }
inE
isF
-linearly independent, thenA
andL
are 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.
IntermediateField.LinearDisjoint.isDomain'
,IntermediateField.LinearDisjoint.exists_field_of_isDomain
: ifA
andB
are field extensions ofF
, thenA ⊗[F] B
is a domain if and only if there exists a field extension ofF
thatA
andB
embed into with linearly disjoint images.IntermediateField.LinearDisjoint.isField_of_forall
,IntermediateField.LinearDisjoint.of_isField'
: ifA
andB
are field extensions ofF
, thenA ⊗[F] B
is a field if and only if for any field extension ofF
thatA
andB
embed into, their images are linearly disjoint.Algebra.TensorProduct.isField_of_isAlgebraic
: ifE
andK
are field extensions ofF
, one of them is algebraic, andE ⊗[F] K
is a domain, thenE ⊗[F] K
is also a field. SeeAlgebra.TensorProduct.isAlgebraic_of_isField
for its converse (in an earlier file).IntermediateField.LinearDisjoint.isField_of_isAlgebraic
,IntermediateField.LinearDisjoint.isField_of_isAlgebraic'
: ifA
andB
are field extensions ofF
, one of them is algebraic, such that they are linearly disjoint (more generally, if there exists a field extension ofF
that they embed into with linearly disjoint images), thenA ⊗[F] B
is a field.
Other main results #
IntermediateField.LinearDisjoint.symm
,IntermediateField.linearDisjoint_comm
: linear disjointness is symmetric.IntermediateField.LinearDisjoint.map
: linear disjointness is preserved by algebra homomorphism.IntermediateField.LinearDisjoint.rank_sup
,IntermediateField.LinearDisjoint.finrank_sup
: ifA
andB
are linearly disjoint, then the rank ofA ⊔ B
is equal to the product of the rank ofA
andB
.IntermediateField.LinearDisjoint.of_finrank_sup
: conversely, ifA
andB
are finite extensions, such that rank ofA ⊔ B
is equal to the product of the rank ofA
andB
, thenA
andB
are linearly disjoint.IntermediateField.LinearDisjoint.of_finrank_coprime
: if the rank ofA
andB
are coprime, thenA
andB
are linearly disjoint.IntermediateField.LinearDisjoint.inf_eq_bot
: ifA
andB
are linearly disjoint, then they are disjoint.IntermediateField.LinearDisjoint.algEquiv_of_isAlgebraic
: linear disjointness is preserved by isomorphisms, provided that one of the field is algebraic.
Tags #
linearly disjoint, linearly independent, tensor product
If A
is an intermediate field of E / F
, and E / L / F
is a field extension tower,
then A
and L
are linearly disjoint, if they are linearly disjoint as subalgebras of E
(Subalgebra.LinearDisjoint
).
Equations
- A.LinearDisjoint L = A.LinearDisjoint (IsScalarTower.toAlgHom F L E).range
Instances For
Two intermediate fields are linearly disjoint if and only if they are linearly disjoint as subalgebras.
Linear disjointness is symmetric.
Linear disjointness is symmetric.
Linear disjointness is symmetric.
Linear disjointness is symmetric.
Linear disjointness of intermediate fields is preserved by algebra homomorphisms.
Linear disjointness of an intermediate field with a tower of field embeddings is preserved by algebra homomorphisms.
Linear disjointness is preserved by algebra homomorphism.
If A
and L
are linearly disjoint, then any F
-linearly independent family on A
remains
linearly independent over L
.
If there exists an F
-basis of A
which remains linearly independent over L
, then
A
and L
are linearly disjoint.
If A
and B
are linearly disjoint, then any F
-linearly independent family on B
remains
linearly independent over A
.
If there exists an F
-basis of B
which remains linearly independent over A
, then
A
and B
are linearly disjoint.
If A
and L
are linearly disjoint, then any F
-linearly independent family on L
remains
linearly independent over A
.
If there exists an F
-basis of L
which remains linearly independent over A
, then
A
and L
are linearly disjoint.
If A
and B
are linearly disjoint, then for any F
-linearly independent families
{ u_i }
, { v_j }
of A
, B
, the products { u_i * v_j }
are linearly independent over F
.
If A
and L
are linearly disjoint, then for any F
-linearly independent families
{ u_i }
, { v_j }
of A
, L
, the products { u_i * v_j }
are linearly independent over F
.
If there are F
-bases { u_i }
, { v_j }
of A
, B
, such that the products
{ u_i * v_j }
are linearly independent over F
, then A
and B
are linearly disjoint.
If there are F
-bases { u_i }
, { v_j }
of A
, L
, such that the products
{ u_i * v_j }
are linearly independent over F
, then A
and L
are linearly disjoint.
Similar to IntermediateField.LinearDisjoint.of_le_right
but this is for abstract fields.
If A
and B
are linearly disjoint, A'
and B'
are contained in A
and B
,
respectively, then A'
and B'
are also linearly disjoint.
Similar to IntermediateField.LinearDisjoint.of_le
but this is for abstract fields.
If A
and A
itself are linearly disjoint over F
, then it is equal to F
.
If A
and B
are linearly disjoint over F
, then the
rank of A ⊔ B
is equal to the product of that of A
and B
.
If A
and B
are linearly disjoint over F
, then the Module.finrank
of
A ⊔ B
is equal to the product of that of A
and B
.
If A
and B
are finite extensions of F
,
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 L
have coprime degree over F
, then they are linearly disjoint.
If A
and L
are linearly disjoint over F
, then A ⊗[F] L
is a domain.
If A
and B
are field extensions of F
, there exists a field extension E
of F
that
A
and B
embed into with linearly disjoint images, then A ⊗[F] B
is a domain.
If A ⊗[F] L
is a field, then A
and L
are linearly disjoint over F
.
If A
and B
are field extensions of F
, such that A ⊗[F] B
is a field, then for any
field extension of F
that A
and B
embed into, their images are linearly disjoint.
If A
and B
are field extensions of F
, such that A ⊗[F] B
is a domain, then there exists
a field extension of F
that A
and B
embed into with linearly disjoint images.
If for any field extension K
of F
that A
and B
embed into, their images are
linearly disjoint, then A ⊗[F] B
is a field. (In the proof we choose K
to be the quotient
of A ⊗[F] B
by a maximal ideal.)
If E
and K
are field extensions of F
, one of them is algebraic, such that
E ⊗[F] K
is a domain, then E ⊗[F] K
is also a field. It is a corollary of
Subalgebra.LinearDisjoint.exists_field_of_isDomain_of_injective
and
IntermediateField.sup_toSubalgebra_of_isAlgebraic
.
See Algebra.TensorProduct.isAlgebraic_of_isField
for its converse (in an earlier file).
If A
and L
are linearly disjoint over F
and one of them is algebraic,
then A ⊗[F] L
is a field.
If A
and B
are field extensions of F
, one of them is algebraic, such that there exists a
field E
that A
and B
embeds into with linearly disjoint images, then A ⊗[F] B
is a field.
If A
and L
are linearly disjoint, one of them is algebraic, then for any B
and L'
isomorphic to A
and L
respectively, B
and L'
are also linearly disjoint.