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
I
of Dedekind domainR
- An
R
-algebraS
that is a Dedekind Domain - An
α : S
such that that is integral overR
with minimal polynomialf
If the conductor𝓒
ofx
is such that𝓒 ∩ R
is coprime toI
then the prime factorisations ofI * S
andf mod I
have the same shape, i.e. they have the same number of prime factors, and each prime factors ofI * S
can be paired with a prime factor off mod I
in 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 * S
and the prime factors off mod I
.
Main results #
normalized_factors_ideal_map_eq_normalized_factors_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, wherepb
is a power basis ofS
overR
.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk_symm_apply_eq_span
: LetQ
be a lift of factor of the minimal polynomial ofx
, a generator ofS
overR
, takenmod I
. Then (the reduction of)Q
corresponds vianormalizedFactorsMapEquivNormalizedFactorsMinPolyMk
tospan (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
This technical lemma tell us that if C
is the conductor of R<x>
and I
is an ideal of R
then p * (I * S) ⊆ I * R<x>
for any p
in C ∩ R
A technical result telling us that (I * S) ∩ R<x> = I * R<x>
for any ideal I
of R
.
The canonical morphism of rings from R<x> ⧸ (I*R<x>)
to S ⧸ (I*S)
is an isomorphism
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 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})
.