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 #
NumberField.InfiniteAdeleRing
of a number fieldK
is defined as the product of the completions ofK
over its infinite places.NumberField.InfiniteAdeleRing.ringEquiv_mixedSpace
is the ring isomorphism between the infinite adele ring ofK
andℝ ^ r₁ × ℂ ^ r₂
, where(r₁, r₂)
is the signature ofK
.NumberField.AdeleRing K
is the adele ring of a number fieldK
.NumberField.AdeleRing.principalSubgroup K
is the subgroup of principal adeles(x)ᵥ
.
Main results #
NumberField.InfiniteAdeleRing.locallyCompactSpace
: the infinite adele ring is a locally compact space.
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
- NumberField.InfiniteAdeleRing K = ((v : NumberField.InfinitePlace K) → v.Completion)
Instances For
Equations
- NumberField.InfiniteAdeleRing.instInhabited K = { default := 0 }
The infinite adele ring is locally compact.
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
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 #
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
Equations
Equations
- NumberField.AdeleRing.instInhabited R K = { default := 0 }
Equations
The subgroup of principal adeles (x)ᵥ
where x ∈ K
.
Equations
- NumberField.AdeleRing.principalSubgroup R K = (algebraMap K (NumberField.AdeleRing R K)).range.toAddSubgroup