Documentation

Mathlib.NumberTheory.NumberField.AdeleRing

The adele ring of a number field #

This file contains the formalisation of the infinite adele ring of a number field as the finite product of completions over its infinite places and the adele ring of a number field as the direct product of the infinite adele ring and the finite adele ring.

Main definitions #

Main results #

References #

Tags #

infinite adele ring, adele ring, number field

The infinite adele ring #

The infinite adele ring is the finite product of completions of a number field over its infinite places. See NumberField.InfinitePlace for the definition of an infinite place and NumberField.InfinitePlace.Completion for the associated completion.

The infinite adele ring of a number field.

Equations
Instances For
    @[simp]

    The infinite adele ring is locally compact.

    @[reducible, inline]

    The ring isomorphism between the infinite adele ring of a number field and the space ℝ ^ r₁ × ℂ ^ r₂, where (r₁, r₂) is the signature of the number field.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem NumberField.InfiniteAdeleRing.ringEquiv_mixedSpace_apply (K : Type u_1) [Field K] (x : InfiniteAdeleRing K) :
      (ringEquiv_mixedSpace K) x = (fun (v : { w : InfinitePlace K // w.IsReal }) => (InfinitePlace.Completion.extensionEmbeddingOfIsReal ) (x v), fun (v : { w : InfinitePlace K // w.IsComplex }) => (InfinitePlace.Completion.extensionEmbedding v) (x v))

      Transfers the embedding of x ↦ (x)ᵥ of the number field K into its infinite adele ring to the mixed embedding x ↦ (φᵢ(x))ᵢ of K into the space ℝ ^ r₁ × ℂ ^ r₂, where (r₁, r₂) is the signature of K and φᵢ are the complex embeddings of K.

      The adele ring #

      def NumberField.AdeleRing (R : Type u_1) (K : Type u_2) [CommRing R] [IsDedekindDomain R] [Field K] [Algebra R K] [IsFractionRing R K] :
      Type (max u_2 u_2 u_1)

      AdeleRing (𝓞 K) K is the adele ring of a number field K.

      More generally AdeleRing R K can be used if K is the field of fractions of the Dedekind domain R. This enables use of rings like AdeleRing ℤ ℚ, which in practice are easier to work with than AdeleRing (𝓞 ℚ) ℚ.

      Note that this definition does not give the correct answer in the function field case.

      Equations
      Instances For
        @[simp]
        theorem NumberField.AdeleRing.algebraMap_fst_apply (R : Type u_1) (K : Type u_2) [CommRing R] [IsDedekindDomain R] [Field K] [Algebra R K] [IsFractionRing R K] (x : K) (v : InfinitePlace K) :
        ((algebraMap K (AdeleRing R K)) x).1 v = x
        @[simp]
        theorem NumberField.AdeleRing.algebraMap_snd_apply (R : Type u_1) (K : Type u_2) [CommRing R] [IsDedekindDomain R] [Field K] [Algebra R K] [IsFractionRing R K] (x : K) (v : IsDedekindDomain.HeightOneSpectrum R) :
        (fun (v : IsDedekindDomain.HeightOneSpectrum R) => ((algebraMap K (AdeleRing R K)) x).2 v) v = x
        @[reducible, inline]

        The subgroup of principal adeles (x)ᵥ where x ∈ K.

        Equations
        Instances For