Kummer-Dedekind theorem #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file proves the monogenic version of the Kummer-Dedekind theorem on the splitting of prime
ideals in an extension of the ring of integers. This states that if I is a prime ideal of
Dedekind domain R and S = R[α] for some α that is integral over R with minimal polynomial
f, then the prime factorisations of I * S and f mod I have the same shape, i.e. they have the
same number of prime factors, and each prime factors of I * S can be paired with a prime factor
of f mod I in a way that ensures multiplicities match (in fact, this pairing can be made explicit
with a formula).
Main definitions #
normalized_factors_map_equiv_normalized_factors_min_poly_mk: 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 #
normalized_factors_ideal_map_eq_normalized_factors_min_poly_mk_map: The Kummer-Dedekind theorem.ideal.irreducible_map_of_irreducible_minpoly:I.map (algebra_map R S)is irreducible if(map I^.quotient.mk (minpoly R pb.gen))is irreducible, wherepbis a power basis ofSoverR.
TODO #
-
Prove the Kummer-Dedekind theorem in full generality.
-
Prove the converse of
ideal.irreducible_map_of_irreducible_minpoly. -
Prove that
normalized_factors_map_equiv_normalized_factors_min_poly_mkcan be expressed asnormalized_factors_map_equiv_normalized_factors_min_poly_mk g = ⟨I, G(α)⟩forga prime factor off mod IandGa lift ofgtoR[X].
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
- quot_adjoin_equiv_quot_map hx h_alg = ring_equiv.of_bijective (ideal.quotient.lift (ideal.map (algebra_map R ↥(algebra.adjoin R {x})) I) ((ideal.quotient.mk (ideal.map (algebra_map R S) I)).comp (algebra_map ↥(algebra.adjoin R {x}) S)) quot_adjoin_equiv_quot_map._proof_1) _
The first half of the Kummer-Dedekind Theorem in the monogenic case, 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
- kummer_dedekind.normalized_factors_map_equiv_normalized_factors_min_poly_mk hI hI' hx hx' = (normalized_factors_equiv_of_quot_equiv ((quot_adjoin_equiv_quot_map hx kummer_dedekind.normalized_factors_map_equiv_normalized_factors_min_poly_mk._proof_16).symm.trans (((algebra.adjoin.power_basis' hx').quotient_equiv_quotient_minpoly_map I).to_ring_equiv.trans (ideal.quot_equiv_of_eq _))) _ _).trans (normalized_factors_equiv_span_normalized_factors _).symm
The second half of the Kummer-Dedekind Theorem in the monogenic case, stating that the
bijection factors_equiv' defined in the first half preserves multiplicities.
The Kummer-Dedekind Theorem.