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 #
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θ
.
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.