Documentation

Mathlib.NumberTheory.NumberField.Completion

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 #

Main results #

Tags #

number field, embeddings, infinite places, completion, absolute value

@[reducible, inline]

The completion of a number field at an infinite place.

Equations
  • v.completion = (↑v).completion
Instances For

    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 →+* ℝ 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
          Instances For

            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
              Instances For