Documentation

Mathlib.NumberTheory.NumberField.CanonicalEmbedding

Canonical embedding of a number field #

The canonical embedding of a number field K of degree n is the ring homomorphism K →+* ℂ^n that sends x ∈ K to (φ_₁(x),...,φ_n(x)) where the φ_i's are the complex embeddings of K. Note that we do not choose an ordering of the embeddings, but instead map K into the type (K →+* ℂ) → ℂ of -vectors indexed by the complex embeddings.

Main definitions and results #

Tags #

number field, infinite places

The canonical embedding of a number field K of degree n into ℂ^n.

Instances For
    @[simp]
    theorem NumberField.canonicalEmbedding.apply_at {K : Type u_1} [Field K] (φ : K →+* ) (x : K) :
    ↑(NumberField.canonicalEmbedding K) x φ = φ x

    The image of canonicalEmbedding lives in the -submodule of the x ∈ ((K →+* ℂ) → ℂ) such that conj x_φ = x_(conj φ) for all ∀ φ : K →+* ℂ.

    The image of 𝓞 K as a subring of ℂ^n.

    Instances For

      A -basis of ℂ^n that is also a -basis of the integerLattice.

      Instances For
        noncomputable def NumberField.mixedEmbedding (K : Type u_1) [Field K] :

        The mixed embedding of a number field K of signature (r₁, r₂) into ℝ^r₁ × ℂ^r₂.

        Instances For

          The linear map that makes canonicalEmbedding and mixedEmbedding commute, see commMap_canonical_eq_mixed.

          Instances For

            This is a technical result to ensure that the image of the -basis of ℂ^n defined in canonicalEmbedding.latticeBasis is a -basis of ℝ^r₁ × ℂ^r₂, see mixedEmbedding.latticeBasis.

            A -basis of ℝ^r₁ × ℂ^r₂ that is also a -basis of the image of 𝓞 K.

            Instances For
              @[inline, reducible]

              The convex body defined by f: the set of points x : E such that ‖x w‖ < f w for all infinite places w.

              Instances For
                @[inline, reducible]

                The fudge factor that appears in the formula for the volume of convexBodyLt.

                Instances For

                  The volume of (ConvexBodyLt K f) where convexBodyLt K f is the set of points x such that ‖x w‖ < f w for all infinite places w.

                  theorem NumberField.mixedEmbedding.adjust_f (K : Type u_1) [Field K] {f : NumberField.InfinitePlace KNNReal} [NumberField K] {w₁ : NumberField.InfinitePlace K} (B : NNReal) (hf : ∀ (w : NumberField.InfinitePlace K), w w₁f w 0) :
                  g, (∀ (w : NumberField.InfinitePlace K), w w₁g w = f w) (Finset.prod Finset.univ fun w => g w ^ NumberField.InfinitePlace.mult w) = B

                  This is a technical result: quite often, we want to impose conditions at all infinite places but one and choose the value at the remaining place so that we can apply exists_ne_zero_mem_ringOfIntegers_lt.

                  The bound that appears in Minkowski Convex Body theorem, see MeasureTheory.exists_ne_zero_mem_lattice_of_measure_mul_two_pow_lt_measure.

                  Instances For

                    Assume that f : InfinitePlace K → ℝ≥0 is such that minkowskiBound K < volume (convexBodyLt K f) where convexBodyLt K f is the set of points x such that ‖x w‖ < f w for all infinite places w (see convexBodyLt_volume for the computation of this volume), then there exists a nonzero algebraic integer a in 𝓞 K such that w a < f w for all infinite places w.