Frobenius elements. #
This file proves a general result in commutative algebra which can be used to define Frobenius elements of Galois groups of local or fields (for example number fields).
KB was alerted to this very general result (which needs no Noetherian or finiteness assumptions on the rings, just on the Galois group) by Joel Riou here https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Uses.20of.20Frobenius.20elements.20in.20mathematics/near/448934112
Mathematical details #
The general commutative algebra result #
This is Theorem 2 in Chapter V, Section 2, number 2 of Bourbaki Alg Comm. It says the following.
Let A → B
be commutative rings and let G
be a finite group acting on B
by ring automorphisms,
such that the G
-invariants of B
are exactly the image of A
.
The two claims of the theorem are:
(i) If P
is a prime ideal of A
then G
acts transitively on the primes of B
above P
.
(ii) If Q
is a prime ideal of B
lying over P
then the canonica map from the stabilizer of Q
in G
to the automorphism group of the residue field extension Frac(B/Q) / Frac(A/P)
is
surjective.
We say "automorphism group" rather than "Galois group" because the extension might not be separable (it is algebraic and normal however, but it can be infinite; however its maximal separable subextension is finite).
This result means that if the inertia group I_Q is trivial and the residue fields are finite, there's a Frobenius element Frob_Q in the stabiliser of Q, and a Frobenius conjugacy class Frob_P in G.
The characteristic polynomial of an element b
of a G
-semiring B
is the polynomial ∏_{g ∈ G} (X - g • b)
(here G
is finite; junk
returned in the infinite case) .
Equations
- MulSemiringAction.CharacteristicPolynomial.F G b = ∏ᶠ (τ : G), (Polynomial.X - Polynomial.C (τ • b))
Instances For
Equations
- MulSemiringAction.CharacteristicPolynomial.instAlgebraPolynomial_fLT = (Polynomial.mapRingHom Algebra.toRingHom).toAlgebra
Instances For
This "splitting" function from B to A will only ever be evaluated on
G-invariant elements of B, and the two key facts about it are
that it lifts such an element to A
, and for reasons of
convenience it lifts 1
to 1
.
Equations
- MulSemiringAction.CharacteristicPolynomial.splitting_of_full hFull b = if b = 1 then 1 else if h : ∀ (σ : G), σ • b = b then ⋯.choose else 37
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Equations
- MulSemiringAction.CharacteristicPolynomial.Mbar P hFull' bbar = Polynomial.map (Ideal.Quotient.mk P) (MulSemiringAction.CharacteristicPolynomial.M hFull' (Ideal.Quotient.out bbar))
Instances For
Equations
- instAlgebraPolynomial_fLT = (Polynomial.mapRingHom Algebra.toRingHom).toAlgebra
Instances For
Equations
- Bourbaki52222.residueFieldExtensionPolynomial G L K x = if x = 0 then (Polynomial.monomial (Nat.card G)) 1 else 37
Instances For
Equations
- Bourbaki52222.y L K = ⋯.choose
Instances For
Equations
- Bourbaki52222.quotientRingAction Q Q' g hg = Q.quotientEquiv Q' (MulSemiringAction.toRingEquiv G B g) ⋯
Instances For
Equations
- Bourbaki52222.quotientAlgebraAction Q P g hg = { toEquiv := (Bourbaki52222.quotientRingAction Q Q g hg).toEquiv, map_mul' := ⋯, map_add' := ⋯, commutes' := ⋯ }
Instances For
Equations
- Bourbaki52222.Pointwise.quotientAlgebraActionMonoidHom Q P = { toFun := fun (gh : ↥(MulAction.stabilizer G Q)) => Bourbaki52222.quotientAlgebraAction Q P ↑gh ⋯, map_one' := ⋯, map_mul' := ⋯ }
Instances For
Equations
- Bourbaki52222.IsFractionRing.algEquiv_lift Q P L K e = { toEquiv := (IsFractionRing.fieldEquivOfRingEquiv e.toRingEquiv).toEquiv, map_mul' := ⋯, map_add' := ⋯, commutes' := ⋯ }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
From Bourbaki Comm Alg, Chapter V.