Kummer-Dedekind criterion for the splitting of prime numbers #
In this file, we give a specialized version of the Kummer-Dedekind criterion for the case of the splitting of rational primes in number fields.
Main definitions #
Let K
be a number field and θ
an algebraic integer of K
.
RingOfIntegers.exponent
: the smallest positive integerd
contained in the conductor ofθ
. It is the smallest integer such thatd • 𝓞 K ⊆ ℤ[θ]
, seeRingOfIntegers.exponent_eq_sInf
.RingOfIntegers.ZModXQuotSpanEquivQuotSpan
: The isomorphism between(ℤ / pℤ)[X] / (minpoly θ)
and𝓞 K / p(𝓞 K)
for a primep
which doesn't divide the exponent ofθ
.NumberField.Ideal.primesOverSpanEquivMonicFactorsMod
: The bijection between the prime ideals ofK
abovep
and the monic irreducible factors ofminpoly ℤ θ
modulop
for a primep
which doesn't divide the exponent ofθ
.
Main results #
NumberField.Ideal.primesOverSpanEquivMonicFactorsMod
: The ideal corresponding to the class ofQ ∈ ℤ[X]
modulop
viaNumberField.Ideal.primesOverSpanEquivMonicFactorsMod
is spanned byp
andQ(θ)
.NumberField.Ideal.inertiaDeg_primesOverSpanEquivMonicFactorsMod_symm_apply
: The residual degree of the ideal corresponding to the class ofQ ∈ ℤ[X]
modulop
viaNumberField.Ideal.primesOverSpanEquivMonicFactorsMod
is equal to the degree ofQ mod p
.NumberField.Ideal.ramificationIdx_primesOverSpanEquivMonicFactorsMod_symm_apply
: The ramification index of the ideal corresponding to the class ofQ ∈ ℤ[X]
modulop
viaNumberField.Ideal.primesOverSpanEquivMonicFactorsMod
is equal to the multiplicity ofQ mod p
inminpoly ℤ θ
.
The smallest positive integer d
contained in the conductor of θ
. It is the smallest integer
such that d • 𝓞 K ⊆ ℤ[θ]
, see exponent_eq_sInf
. It is set to 0
if d
does not exists.
Equations
Instances For
If p
doesn't divide the exponent of θ
, then (ℤ / pℤ)[X] / (minpoly θ) ≃+* 𝓞 K / p(𝓞 K)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The finite set of monic irreducible factors of minpoly ℤ θ
modulo p
.
Equations
Instances For
If p
does not divide exponent θ
and Q
is a lift of a monic irreducible factor of
minpoly ℤ θ
modulo p
, then (ℤ / pℤ)[X] / Q ≃+* 𝓞 K / (p, Q(θ))
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If p
does not divide exponent θ
, then the prime ideals above p
in K
are in bijection
with the monic irreducible factors of minpoly ℤ θ
modulo p
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The ideal corresponding to the class of Q ∈ ℤ[X]
modulo p
via
NumberField.Ideal.primesOverSpanEquivMonicFactorsMod
is spanned by p
and Q(θ)
.
The residual degree of the ideal corresponding to the class of Q ∈ ℤ[X]
modulo p
via
NumberField.Ideal.primesOverSpanEquivMonicFactorsMod
is equal to the degree of Q mod p
.
The ramification index of the ideal corresponding to the class of Q ∈ ℤ[X]
modulo p
via
NumberField.Ideal.primesOverSpanEquivMonicFactorsMod
is equal to the multiplicity of Q mod p
in
minpoly ℤ θ
.