Adjoining Elements to Fields #
This file contains many results about adjoining elements to fields.
If E1
and E2
are intermediate fields, and at least one them are algebraic, then the rank of
the compositum of E1
and E2
is less than or equal to the product of that of E1
and E2
.
Note that this result is also true without algebraic assumption,
but the proof becomes very complicated.
If E1
and E2
are intermediate fields, then the Module.finrank
of
the compositum of E1
and E2
is less than or equal to the product of that of E1
and E2
.
A compositum of splitting fields is a splitting field
If K / E / F
is a field extension tower, L
is an intermediate field of K / F
, such that
either E / F
or L / F
is algebraic, then [E(L) : E] ≤ [L : F]
. A corollary of
Subalgebra.adjoin_rank_le
since in this case E(L) = E[L]
.
If F⟮x⟯
has dimension ≤1
over F
for every x ∈ E
then F = E
.
algebra isomorphism between AdjoinRoot
and F⟮α⟯
Stacks Tag 09G1 (Algebraic case)
Equations
Instances For
The elements 1, x, ..., x ^ (d - 1)
form a basis for K⟮x⟯
,
where d
is the degree of the minimal polynomial of x
.
Equations
- IntermediateField.powerBasisAux hx = (AdjoinRoot.powerBasis ⋯).basis.map (IntermediateField.adjoinRootEquivAdjoin K hx).toLinearEquiv
Instances For
The power basis 1, x, ..., x ^ (d - 1)
for K⟮x⟯
,
where d
is the degree of the minimal polynomial of x
.
Equations
- IntermediateField.adjoin.powerBasis hx = { gen := IntermediateField.AdjoinSimple.gen K x, dim := (minpoly K x).natDegree, basis := IntermediateField.powerBasisAux hx, basis_eq_pow := ⋯ }
Instances For
If x
is an algebraic element of field K
, then its minimal polynomial has degree
[K(x) : K]
.
If K / E / F
is a field extension tower, S ⊂ K
is such that F(S) = K
,
then E(S) = K
.
If E / F
is a finite extension such that E = F(α)
, then for any intermediate field K
, the
F
adjoin the coefficients of minpoly K α
is equal to K
itself.
If E / F
is an infinite algebraic extension, then there exists an intermediate field
L / F
with arbitrarily large finite extension degree.
If x : L
is an integral element in a field extension L
over K
, then the degree of the
minimal polynomial of x
over K
divides [L : K]
.
A compositum of algebraic extensions is algebraic
If L / K
is a field extension, S
is a finite subset of L
, such that every element of S
is integral (= algebraic) over K
, then K(S) / K
is a finite extension.
A direct corollary of finiteDimensional_iSup_of_finite
.
Algebra homomorphism F⟮α⟯ →ₐ[F] K
are in bijection with the set of roots
of minpoly α
in K
.
Equations
- IntermediateField.algHomAdjoinIntegralEquiv F h = (IntermediateField.adjoin.powerBasis h).liftEquiv'.trans ((Equiv.refl K).subtypeEquiv ⋯)
Instances For
Fintype of algebra homomorphism F⟮α⟯ →ₐ[F] K
Equations
Instances For
Let f, g
be monic polynomials over K
. If f
is irreducible, and g(x) - α
is irreducible
in K⟮α⟯
with α
a root of f
, then f(g(x))
is irreducible.
The canonical algebraic homomorphism from AdjoinRoot p
to AdjoinRoot q
, where
the polynomial q : K[X]
divides p
.
Equations
- AdjoinRoot.algHomOfDvd hpq = AdjoinRoot.liftHom p (AdjoinRoot.root q) ⋯
Instances For
algHomOfDvd
sends AdjoinRoot.root p
to AdjoinRoot.root q
.
The canonical algebraic equivalence between AdjoinRoot p
and AdjoinRoot q
, where
the two polynomials p q : K[X]
are equal.
Equations
- AdjoinRoot.algEquivOfEq hp h_eq = AlgEquiv.ofAlgHom (AdjoinRoot.algHomOfDvd ⋯) (AdjoinRoot.algHomOfDvd ⋯) ⋯ ⋯
Instances For
algEquivOfEq
sends AdjoinRoot.root p
to AdjoinRoot.root q
.
The canonical algebraic equivalence between AdjoinRoot p
and AdjoinRoot q
,
where the two polynomials p q : K[X]
are associated.
Equations
- AdjoinRoot.algEquivOfAssociated hp hpq = AlgEquiv.ofAlgHom (AdjoinRoot.liftHom p (AdjoinRoot.root q) ⋯) (AdjoinRoot.liftHom q (AdjoinRoot.root p) ⋯) ⋯ ⋯
Instances For
algEquivOfAssociated
sends AdjoinRoot.root p
to AdjoinRoot.root q
.
The canonical algEquiv
between K⟮x⟯
and K⟮y⟯
, sending x
to y
, where x
and y
have
the same minimal polynomial over K
.
Equations
- minpoly.algEquiv hx h_mp = (IntermediateField.adjoinRootEquivAdjoin K ⋯).symm.trans ((AdjoinRoot.algEquivOfEq ⋯ h_mp).trans (IntermediateField.adjoinRootEquivAdjoin K ⋯))
Instances For
minpoly.algEquiv
sends the generator of K⟮x⟯
to the generator of K⟮y⟯
.
pb.equivAdjoinSimple
is the equivalence between K⟮pb.gen⟯
and L
itself.
Equations
- pb.equivAdjoinSimple = (IntermediateField.adjoin.powerBasis ⋯).equivOfMinpoly pb ⋯