Kummer-Dedekind theorem #
This file proves the Kummer-Dedekind theorem on the splitting of prime ideals in an extension of the ring of integers. This states the following: assume we are given
- A prime ideal
Iof Dedekind domainR - An
R-algebraSthat is a Dedekind Domain - An
α : Sthat is integral overRwith minimal polynomialfIf the conductor𝓒ofxis such that𝓒 ∩ Ris coprime toIthen the prime factorisations ofI * Sandf mod Ihave the same shape, i.e. they have the same number of prime factors, and each prime factors ofI * Scan be paired with a prime factor off mod Iin a way that ensures multiplicities match (in fact, this pairing can be made explicit with a formula).
Main definitions #
normalizedFactorsMapEquivNormalizedFactorsMinPolyMk: The bijection in the Kummer-Dedekind theorem. This is the pairing between the prime factors ofI * Sand the prime factors off mod I.
Main results #
normalizedFactors_ideal_map_eq_normalizedFactors_min_poly_mk_map: The Kummer-Dedekind theorem.Ideal.irreducible_map_of_irreducible_minpoly:I.map (algebraMap R S)is irreducible if(map (Ideal.Quotient.mk I) (minpoly R pb.gen))is irreducible, wherepbis a power basis ofSoverR.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk_symm_apply_eq_span: LetQbe a lift of factor of the minimal polynomial ofx, a generator ofSoverR, takenmod I. Then (the reduction of)Qcorresponds vianormalizedFactorsMapEquivNormalizedFactorsMinPolyMktospan (I.map (algebraMap R S) ∪ {Q.aeval x}).
TODO #
- Prove the converse of
Ideal.irreducible_map_of_irreducible_minpoly.
References #
Tags #
kummer, dedekind, kummer dedekind, dedekind-kummer, dedekind kummer
The isomorphism of rings between S / I and (R / I)[X] / minpoly x when I
and (conductor R x) ∩ R are coprime.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The first half of the Kummer-Dedekind Theorem, stating that the prime
factors of I*S are in bijection with those of the minimal polynomial of the generator of S
over R, taken mod I.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The second half of the Kummer-Dedekind Theorem, stating that the
bijection FactorsEquiv' defined in the first half preserves multiplicities.
The Kummer-Dedekind Theorem.
Let Q be a lift of factor of the minimal polynomial of x, a generator of S over R, taken
mod I. Then (the reduction of) Q corresponds via
normalizedFactorsMapEquivNormalizedFactorsMinPolyMk to
span (I.map (algebraMap R S) ∪ {Q.aeval x}).