The completion of a number field at an infinite place #
This file contains the completion of a number field at an infinite place. This is ultimately
achieved by applying the UniformSpace.Completion
functor, however each infinite place induces
its own UniformSpace
instance on the number field, so the inference system cannot automatically
infer these. A common approach to handle the ambiguity that arises from having multiple sources
of instances is through the use of type synonyms. In this case, we use the type synonym WithAbs
of a semiring. In particular this type synonym depends on an absolute value, which provides a
systematic way of assigning and inferring instances of the semiring that also depend on an absolute
value. The completion of a field at multiple absolute values is defined in
Mathlib.Algebra.Ring.WithAbs
as AbsoluteValue.completion
. The completion of a number
field at an infinite place is then derived in this file, as InfinitePlace
is a subtype of
AbsoluteValue
.
Main definitions #
NumberField.InfinitePlace.completion
: the completion of a number fieldK
at an infinite place, obtained by completingK
with respect to the absolute value associated to the infinite place.NumberField.InfinitePlace.Completion.extensionEmbedding
: the embeddingv.embedding : K →+* ℂ
extended tov.completion →+* ℂ
.NumberField.InfinitePlace.Completion.extensionEmbedding_of_isReal
: if the infinite placev
is real, then this extends the embeddingv.embedding_of_isReal : K →+* ℝ
tov.completion →+* ℝ
.NumberField.InfinitePlace.Completion.equiv_real_of_isReal
: the ring isomorphismv.completion ≃+* ℝ
whenv
is a real infinite place; the forward direction of this isextensionEmbedding_of_isReal
.NumberField.InfinitePlace.Completion.equiv_complex_of_isComplex
: the ring isomorphismv.completion ≃+* ℂ
whenv
is a complex infinite place; the forward direction of this isextensionEmbedding
.
Main results #
NumberField.Completion.locallyCompactSpace
: the completion of a number field at an infinite place is locally compact.NumberField.Completion.isometry_extensionEmbedding
: the embeddingv.completion →+* ℂ
is an isometry. See alsoisometry_extensionEmbedding_of_isReal
for the corresponding result onv.completion →+* ℝ
whenv
is real.NumberField.Completion.bijective_extensionEmbedding_of_isComplex
: the embeddingv.completion →+* ℂ
is bijective whenv
is complex. See alsobijective_extensionEmebdding_of_isReal
for the corresponding result forv.completion →+* ℝ
whenv
is real.
Tags #
number field, embeddings, infinite places, completion, absolute value
The completion of a number field at an infinite place.
Equations
- v.completion = (↑v).completion
Instances For
Equations
- NumberField.InfinitePlace.Completion.instAlgebraCompletion v = inferInstanceAs (Algebra (WithAbs ↑v) (↑v).completion)
The completion of a number field at an infinite place is locally compact.
Equations
- ⋯ = ⋯
The embedding associated to an infinite place extended to an embedding v.completion →+* ℂ
.
Equations
Instances For
The embedding K →+* ℝ
associated to a real infinite place extended to v.completion →+* ℝ
.
Equations
Instances For
The embedding v.completion →+* ℂ
is an isometry.
The embedding v.completion →+* ℝ
at a real infinite palce is an isometry.
The embedding v.completion →+* ℂ
has closed image inside ℂ
.
The embedding v.completion →+* ℝ
associated to a real infinite place has closed image
inside ℝ
.
If v
is a complex infinite place, then the embedding v.completion →+* ℂ
is surjective.
If v
is a complex infinite place, then the embedding v.completion →+* ℂ
is bijective.
The ring isomorphism v.completion ≃+* ℂ
, when v
is complex, given by the bijection
v.completion →+* ℂ
.
Equations
Instances For
If the infinite place v
is complex, then v.completion
is isometric to ℂ
.
Equations
- NumberField.InfinitePlace.Completion.isometryEquiv_complex_of_isComplex hv = { toEquiv := ↑(NumberField.InfinitePlace.Completion.ringEquiv_complex_of_isComplex hv), isometry_toFun := ⋯ }
Instances For
If v
is a real infinite place, then the embedding v.completion →+* ℝ
is surjective.
If v
is a real infinite place, then the embedding v.completion →+* ℝ
is bijective.
The ring isomorphism v.completion ≃+* ℝ
, when v
is real, given by the bijection
v.completion →+* ℝ
.
Equations
Instances For
If the infinite place v
is real, then v.completion
is isometric to ℝ
.
Equations
- NumberField.InfinitePlace.Completion.isometryEquiv_real_of_isReal hv = { toEquiv := ↑(NumberField.InfinitePlace.Completion.ringEquiv_real_of_isReal hv), isometry_toFun := ⋯ }