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.instCommRing K = Pi.commRing
Equations
- NumberField.InfiniteAdeleRing.instInhabited K = { default := 0 }
Equations
- ⋯ = ⋯
Equations
- NumberField.InfiniteAdeleRing.instTopologicalSpace K = Pi.topologicalSpace
Equations
- ⋯ = ⋯
Equations
- NumberField.InfiniteAdeleRing.instAlgebra K = Pi.algebra (NumberField.InfinitePlace K) NumberField.InfinitePlace.completion
The infinite adele ring is locally compact.
Equations
- ⋯ = ⋯
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 #
The adele ring of a number field.
Equations
Instances For
Equations
- NumberField.AdeleRing.instCommRing K = Prod.instCommRing
Equations
- NumberField.AdeleRing.instInhabited K = { default := 0 }
Equations
- NumberField.AdeleRing.instTopologicalSpace K = instTopologicalSpaceProd
Equations
- ⋯ = ⋯
The subgroup of principal adeles (x)ᵥ
where x ∈ K
.
Equations
- NumberField.AdeleRing.principalSubgroup K = (algebraMap K (NumberField.AdeleRing K)).range.toAddSubgroup