Documentation

Mathlib.NumberTheory.NumberField.FinitePlaces

Finite places of number fields #

This file defines finite places of a number field K as absolute values coming from an embedding into a completion of K associated to a non-zero prime ideal of š“ž K.

Main Definitions and Results #

Tags #

number field, places, finite places

theorem NumberField.one_lt_norm {K : Type u_1} [Field K] [NumberField K] (v : IsDedekindDomain.HeightOneSpectrum (NumberField.RingOfIntegers K)) :
1 < ā†‘(Ideal.absNorm v.asIdeal)

The norm of a maximal ideal as an element of ā„ā‰„0 is > 1

The v-adic absolute value on K defined as the norm of v raised to negative v-adic valuation.

Equations
Instances For

    The embedding of a number field inside its completion with respect to v.

    Equations
    Instances For
      Equations

      A finite place of a number field K is a place associated to an embedding into a completion with respect to a maximal ideal.

      Equations
      Instances For

        Return the finite place defined by a maximal ideal v.

        Equations
        Instances For

          The norm of the image after the embedding associated to v is equal to the v-adic absolute value.

          The norm of the image after the embedding associated to v is equal to the norm of v raised to the power of the v-adic valuation.

          The norm of the image after the embedding associated to v is equal to the norm of v raised to the power of the v-adic valuation for integers.

          The v-adic norm of an integer is 1 if and only if it is not in the ideal.

          The v-adic norm of an integer is less than 1 if and only if it is in the ideal.

          Equations
          • NumberField.FinitePlace.instFunLikeReal = { coe := fun (w : NumberField.FinitePlace K) (x : K) => ā†‘w x, coe_injective' := ā‹Æ }

          For a finite place w, return a maximal ideal v such that w = finite_place v .

          Equations
          • w.maximalIdeal = ā‹Æ.choose
          Instances For
            theorem NumberField.FinitePlace.maximalIdeal_inj {K : Type u_1} [Field K] [NumberField K] (wā‚ wā‚‚ : NumberField.FinitePlace K) :
            wā‚.maximalIdeal = wā‚‚.maximalIdeal ā†” wā‚ = wā‚‚
            theorem NumberField.FinitePlace.mulSupport_finite {K : Type u_1} [Field K] [NumberField K] {x : K} (h_x_nezero : x ā‰  0) :
            (Function.mulSupport fun (w : NumberField.FinitePlace K) => w x).Finite