The topological abelianization of the absolute Galois group. #
We define the absolute Galois group of a field K
and its topological abelianization.
Main definitions #
Field.absoluteGaloisGroup
: The Galois group of the field extensionK^al/K
, whereK^al
is an algebraic closure ofK
.Field.absoluteGaloisGroupAbelianization
: The topological abelianization ofField.absoluteGaloisGroup K
, that is, the quotient ofField.absoluteGaloisGroup K
by the topological closure of its commutator subgroup.
Main results #
Field.absoluteGaloisGroup.commutator_closure_isNormal
: the topological closure of the commutator ofabsoluteGaloisGroup
is a normal subgroup.
Tags #
field, algebraic closure, galois group, abelianization
The absolute Galois group #
The absolute Galois group of K
, defined as the Galois group of the field extension K^al/K
,
where K^al
is an algebraic closure of K
.
Equations
Instances For
Equations
- Field.instGroupAbsoluteGaloisGroup K = AlgEquiv.aut
absoluteGaloisGroup
is a topological space with the Krull topology.
Equations
The topological abelianization of the absolute Galois group #
instance
Field.absoluteGaloisGroup.commutator_closure_isNormal
(K : Type u_1)
[Field K]
:
(commutator (Field.absoluteGaloisGroup K)).topologicalClosure.Normal
Equations
- ⋯ = ⋯
@[reducible, inline]
The topological abelianization of absoluteGaloisGroup
, that is, the quotient of
absoluteGaloisGroup
by the topological closure of its commutator subgroup.