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
    @[deprecated NumberField.InfinitePlace.Completion]

    Alias of NumberField.InfinitePlace.Completion.


    The completion of a number field at an infinite place.

    Equations
    Instances For

      The coercion from the rationals to its completion along an infinite place is Rat.cast.

      The completion of a number field at an infinite place is locally compact.

      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
          @[deprecated NumberField.InfinitePlace.Completion.extensionEmbeddingOfIsReal]

          Alias of NumberField.InfinitePlace.Completion.extensionEmbeddingOfIsReal.


          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
              @[deprecated NumberField.InfinitePlace.Completion.ringEquivComplexOfIsComplex]

              Alias of NumberField.InfinitePlace.Completion.ringEquivComplexOfIsComplex.


              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
                  @[deprecated NumberField.InfinitePlace.Completion.isometryEquivComplexOfIsComplex]

                  Alias of NumberField.InfinitePlace.Completion.isometryEquivComplexOfIsComplex.


                  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
                      @[deprecated NumberField.InfinitePlace.Completion.ringEquivRealOfIsReal]

                      Alias of NumberField.InfinitePlace.Completion.ringEquivRealOfIsReal.


                      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
                          @[deprecated NumberField.InfinitePlace.Completion.isometryEquivRealOfIsReal]

                          Alias of NumberField.InfinitePlace.Completion.isometryEquivRealOfIsReal.


                          If the infinite place v is real, then v.Completion is isometric to .

                          Equations
                          Instances For