Adjoining Elements to Fields #
In this file we introduce the notion of adjoining elements to fields.
This isn't quite the same as adjoining elements to rings.
For example, Algebra.adjoin K {x}
might not include x⁻¹
.
Notation #
F⟮α⟯
: adjoin a single elementα
toF
(in scopeIntermediateField
).
adjoin F S
extends a field F
by adjoining a set S ⊆ E
.
Stacks Tag 09FZ (first part)
Equations
- IntermediateField.adjoin F S = { toSubsemiring := (Subfield.closure (Set.range ⇑(algebraMap F E) ∪ S)).toSubsemiring, algebraMap_mem' := ⋯, inv_mem' := ⋯ }
Instances For
Galois insertion between adjoin
and coe
.
Equations
- IntermediateField.gi = { choice := fun (s : Set E) (hs : ↑(IntermediateField.adjoin F s) ≤ s) => (IntermediateField.adjoin F s).copy s ⋯, gc := ⋯, le_l_u := ⋯, choice_eq := ⋯ }
Instances For
Equations
- IntermediateField.instCompleteLattice = CompleteLattice.mk ⋯ ⋯ ⋯ ⋯ ⋯ ⋯
Equations
- IntermediateField.instInhabited = { default := ⊤ }
Equations
- IntermediateField.instUnique = { toInhabited := inferInstanceAs (Inhabited (IntermediateField F F)), uniq := ⋯ }
Construct an algebra isomorphism from an equality of intermediate fields
Equations
- IntermediateField.equivOfEq h = S.equivOfEq T.toSubalgebra ⋯
Instances For
The bottom intermediate_field is isomorphic to the field.
Equations
- IntermediateField.botEquiv F E = (⊥.equivOfEq ⊥ ⋯).trans (Algebra.botEquiv F E)
Instances For
Equations
- IntermediateField.algebraOverBot = (↑(IntermediateField.botEquiv F E)).toAlgebra
The top IntermediateField
is isomorphic to the field.
This is the intermediate field version of Subalgebra.topEquiv
.
Instances For
An intermediate field is isomorphic to its image under an AlgHom
(which is automatically injective)
Equations
- L.equivMap f = (AlgEquiv.ofInjective (f.comp L.val) ⋯).trans (IntermediateField.equivOfEq ⋯)
Instances For
Equations
- IntermediateField.adjoin.fieldCoe F S = { coe := fun (x : F) => ⟨(algebraMap F E) x, ⋯⟩ }
F[S][T] = F[T][S]
If E / L / F
and E / L' / F
are two field extension towers, L ≃ₐ[F] L'
is an isomorphism
compatible with E / L
and E / L'
, then for any subset S
of E
, L(S)
and L'(S)
are
equal as intermediate fields of E / F
.
If x₁ x₂ ... xₙ : E
then F⟮x₁,x₂,...,xₙ⟯
is the IntermediateField F E
generated by these elements.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
generator of F⟮α⟯
Equations
- IntermediateField.AdjoinSimple.gen F α = ⟨α, ⋯⟩
Instances For
An intermediate field S
is finitely generated if there exists t : Finset E
such that
IntermediateField.adjoin F t = S
.
Stacks Tag 09FZ (second part)
Equations
- S.FG = ∃ (t : Finset E), IntermediateField.adjoin F ↑t = S