Documentation

Mathlib.NumberTheory.NumberField.CMField

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 #

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⁺.

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
    Instances For
      theorem NumberField.IsCMField.exists_isConj (K : Type u_1) [Field K] [NumberField K] [IsCMField K] (φ : K →+* ) :
      ∃ (σ : Gal(K/(maximalRealSubfield K))), ComplexEmbedding.IsConj φ σ
      theorem NumberField.IsCMField.isConj_eq_isConj (K : Type u_1) [Field K] [NumberField K] [IsCMField K] {φ ψ : K →+* } {σ τ : Gal(K/(maximalRealSubfield K))} ( : ComplexEmbedding.IsConj φ σ) ( : ComplexEmbedding.IsConj ψ τ) :
      σ = τ

      All the conjugations of a CM-field over its maximal real subfield are the same.

      noncomputable def NumberField.IsCMField.complexConj (K : Type u_1) [Field K] [NumberField K] [IsCMField K] :
      Gal(K/(maximalRealSubfield K))

      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.

        @[simp]
        theorem NumberField.IsCMField.complexEmbedding_complexConj (K : Type u_1) [Field K] [NumberField K] [IsCMField K] (φ : K →+* ) (x : K) :
        φ ((complexConj K) x) = (starRingEnd ) (φ x)
        @[simp]
        theorem NumberField.IsCMField.infinitePlace_complexConj (K : Type u_1) [Field K] [NumberField K] [IsCMField K] (w : InfinitePlace K) (x : K) :
        w ((complexConj K) x) = w x

        The complex conjugation is an automorphism of degree 2.

        The complex conjugation generates the Galois group of K/K⁺.

        @[simp]

        An element of K is fixed by the complex conjugation iff it lies in K⁺.

        noncomputable instance NumberField.IsCMField.starRing (K : Type u_1) [Field K] [NumberField K] [IsCMField K] :
        Equations
        @[reducible, inline]

        A variant of the complex conjugation defined as an AlgEquiv on the ring of integers.

        Equations
        Instances For
          @[reducible, inline]

          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
              @[simp]

              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
                @[reducible, inline]
                noncomputable abbrev NumberField.IsCMField.indexRealUnits (K : Type u_1) [Field K] [NumberField K] :

                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.

                      theorem NumberField.IsCMField.of_forall_isConj (K : Type u_2) [Field K] [NumberField K] [IsTotallyComplex K] {σ : Gal(K/)} ( : ∀ (φ : K →+* ), ComplexEmbedding.IsConj φ σ) :

                      A totally complex field that has a unique complex conjugation is CM.

                      A totally complex abelian extension of is CM.