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 of K.

Main definitions #

Implementation note #

Most result are proved under the general hypothesis: K/F quadratic extension of number fields with F totally real and K totally complex and then, if relevant, we deduce the special case F = maximalRealSubfield K. Results of the first kind live in the NumberField.CMExtension namespace whereas results of the second kind live in the NumberField.IsCMField namespace.

theorem NumberField.CMExtension.isConj_eq_isConj (F : Type u_1) {K : Type u_2} [Field F] [NumberField F] [Field K] [NumberField K] [IsTotallyComplex K] [Algebra F K] [Algebra.IsQuadraticExtension F K] {φ ψ : K →+* } {σ τ : K ≃ₐ[F] K} ( : ComplexEmbedding.IsConj φ σ) ( : ComplexEmbedding.IsConj ψ τ) :
σ = τ

All the conjugations of a CM-extension are the same.

The complex conjugation of a CM-extension.

Equations
Instances For

    The complex conjugation is the conjugation of any complex embedding of a CM-extension.

    The complex conjugation is an automorphism of degree 2.

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

    A number field K is CM if K is a totally complex quadratic extension of its maximal real subfield.

    Instances
      noncomputable instance NumberField.IsCMField.starRing (K : Type u_1) [Field K] [NumberField K] [IsTotallyComplex K] [IsCMField K] :
      Equations