CM-extension of number fields #
A CM-extension K/F of number fields is an extension where K is totally complex, F is
totally real and K is a quadratic extension of F. In this situation, the totally real
subfield F is (isomorphic to) the maximal real subfield K⁺ of K.
Main definitions and results #
NumberField.IsCMField: A predicate that says that if a number field is CM, then it is a totally complex quadratic extension of its totally real subfieldNumberField.CMExtension.equivMaximalRealSubfield: Any fieldFsuch thatK/Fis a CM-extension is isomorphic to the maximal real subfieldK⁺ofK.NumberField.CMExtension.complexConj_eq_self_iff: all the elements ofKfixed by the complex conjugation come from the maximal real subfieldF.NumberField.CMExtension.indexRealUnits_eq_one_or_two: the index of the subgroup of(𝓞 K)ˣgenerated by the real units and the roots of unity is equal to1or2(seeNumberField.IsCMField.indexRealUnits_eq_two_ifffor the computation of this index).NumberField.IsCMField.regulator_div_regulator_eq_two_pow_mul_indexRealUnits_inv: ratio of regulators ofKandK⁺.NumberField.IsCM.ofIsCMExtension: Assume that there existsFsuch thatK/Fis a CM-extension. ThenKis CM.NumberField.IsCMField.of_isMulCommutative: A totally complex abelian extension ofℚis CM.
Implementation note #
Most results are proved for the case of a CM field, that is K is totally complex quadratic
extension of its totally real. These results live in the NumberField.IsCMField namespace. Some
results deal with the general case K/F, where K is totally complex, F is totally real and
K is a quadratic extension of F, and live in the NumberField.CMExtension namespace. Note that
results for the general case can be deduced for the CM case by using the isomorphism
equivMaximalRealSubfield between F and K⁺ mentioned above.
A number field K is CM if K is a totally complex quadratic extension of its maximal
real subfield K⁺.
- to_isTotallyComplex : IsTotallyComplex K
- is_quadratic : Algebra.IsQuadraticExtension (↥(maximalRealSubfield K)) K
Instances
The equiv between the infinite places of K and the infinite places of K⁺ induced by the
restriction to K⁺, see equivInfinitePlace_apply.
Equations
- NumberField.IsCMField.equivInfinitePlace K = Equiv.ofBijective (fun (w : NumberField.InfinitePlace K) => w.comap (algebraMap (↥(NumberField.maximalRealSubfield K)) K)) ⋯
Instances For
All the conjugations of a CM-field over its maximal real subfield are the same.
The complex conjugation of the CM-field K.
Equations
Instances For
The complex conjugation is the conjugation of any complex embedding of a CM-field.
The complex conjugation is an automorphism of degree 2.
The complex conjugation generates the Galois group of K/K⁺.
An element of K is fixed by the complex conjugation iff it lies in K⁺.
Equations
- NumberField.IsCMField.starRing K = { star := ⇑(NumberField.IsCMField.complexConj K), star_involutive := ⋯, star_mul := ⋯, star_add := ⋯ }
A variant of the complex conjugation defined as an AlgEquiv on the ring of integers.
Equations
Instances For
The complex conjugation as an isomorphism of the units of K.
Equations
Instances For
The subgroup of (𝓞 K)ˣ generated by the units of K⁺. These units are exactly the units fixed
by the complex conjugation, see IsCMField.unitsComplexConj_eq_self_iff.
Equations
Instances For
The image of a root of unity by the complex conjugation is its inverse.
This is the version of Complex.conj_rootsOfUnity for CM-fields.
The map (𝓞 K)ˣ →* torsion K defined by u ↦ u * (conj u)⁻¹.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The action of unitsMulComplexConjInv of the torsion is the same as the 2-power map.
The kernel of unitsMulComplexConjInv is the subgroup of real units.
The index of the image of unitsMulComplexConjInv divides 2.
The index of the subgroup of (𝓞 K)ˣ generated by the real units and the roots of unity. This
index is equal to 1 or 2, see indexRealUnits_eq_one_or_two and indexRealUnits_eq_two_iff.
Equations
Instances For
The index of the subgroup of (𝓞 K)ˣ generated by the real units and the roots of unity is
equal to 1 or 2 (see NumberField.IsCMField.indexRealUnits_eq_two_iff for the computation
of this index).
The index of the subgroup of (𝓞 K)ˣ generated by the real units and the roots of unity is equal
to 2 iff there exists a unit whose image by unitsMulComplexConjInv generates the torsion
subgroup of K.
The fundamental system of units of K⁺ as a family of (𝓞 K)ˣ.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Any field F such that K/F is a CM-extension is isomorphic to the maximal real subfield of K.
Equations
Instances For
If K/F is a CM-extension then K is a CM-field.
A totally complex field that has a unique complex conjugation is CM.
A totally complex abelian extension of ℚ is CM.