Documentation

Mathlib.Analysis.Normed.Ring.WithAbs

WithAbs #

WithAbs v is a type synonym for a semiring R which depends on an absolute value. The point of this is to allow the type class inference system to handle multiple sources of instances that arise from absolute values. See NumberTheory.NumberField.Completion for an example of this being used to define Archimedean completions of a number field.

Main definitions #

def WithAbs {R : Type u_1} {S : Type u_2} [Semiring R] [OrderedSemiring S] :
AbsoluteValue R SType u_1

Type synonym for a semiring which depends on an absolute value. This is a function that takes an absolute value on a semiring and returns the semiring. We use this to assign and infer instances on a semiring that depend on absolute values.

Equations
Instances For
    def WithAbs.equiv {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) :

    Canonical equivalence between WithAbs v and R.

    Equations
    Instances For
      Equations
      • =
      Equations
      instance WithAbs.normedRing {R : Type u_4} [Ring R] (v : AbsoluteValue R ) :
      Equations
      instance WithAbs.normedField {K : Type u_3} [Field K] (v : AbsoluteValue K ) :
      Equations

      WithAbs.equiv preserves the ring structure.

      @[simp]
      theorem WithAbs.equiv_zero {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) :
      @[simp]
      theorem WithAbs.equiv_symm_zero {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) :
      (WithAbs.equiv v).symm 0 = 0
      @[simp]
      theorem WithAbs.equiv_add {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) (x y : WithAbs v) :
      @[simp]
      theorem WithAbs.equiv_symm_add {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) (r s : R) :
      (WithAbs.equiv v).symm (r + s) = (WithAbs.equiv v).symm r + (WithAbs.equiv v).symm s
      @[simp]
      theorem WithAbs.equiv_sub {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) (x y : WithAbs v) [Ring R] :
      @[simp]
      theorem WithAbs.equiv_symm_sub {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) (r s : R) [Ring R] :
      (WithAbs.equiv v).symm (r - s) = (WithAbs.equiv v).symm r - (WithAbs.equiv v).symm s
      @[simp]
      theorem WithAbs.equiv_neg {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) (x : WithAbs v) [Ring R] :
      @[simp]
      theorem WithAbs.equiv_symm_neg {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) (r : R) [Ring R] :
      (WithAbs.equiv v).symm (-r) = -(WithAbs.equiv v).symm r
      @[simp]
      theorem WithAbs.equiv_mul {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) (x y : WithAbs v) :
      @[simp]
      theorem WithAbs.equiv_symm_mul {R : Type u_1} [Semiring R] (v : AbsoluteValue R ) (x y : WithAbs v) :
      (WithAbs.equiv v).symm (x * y) = (WithAbs.equiv v).symm x * (WithAbs.equiv v).symm y

      WithAbs.equiv as a ring equivalence.

      Equations
      Instances For

        The completion of a field at an absolute value.

        theorem WithAbs.isometry_of_comp {K : Type u_4} [Field K] {v : AbsoluteValue K } {L : Type u_5} [NormedField L] {f : WithAbs v →+* L} (h : ∀ (x : WithAbs v), f x = v x) :

        If the absolute value v factors through an embedding f into a normed field, then f is an isometry.

        theorem WithAbs.pseudoMetricSpace_induced_of_comp {K : Type u_4} [Field K] {v : AbsoluteValue K } {L : Type u_5} [NormedField L] {f : WithAbs v →+* L} (h : ∀ (x : WithAbs v), f x = v x) :
        PseudoMetricSpace.induced (⇑f) inferInstance = MetricSpace.toPseudoMetricSpace

        If the absolute value v factors through an embedding f into a normed field, then the pseudo metric space associated to the absolute value is the same as the pseudo metric space induced by f.

        theorem WithAbs.uniformSpace_comap_eq_of_comp {K : Type u_4} [Field K] {v : AbsoluteValue K } {L : Type u_5} [NormedField L] {f : WithAbs v →+* L} (h : ∀ (x : WithAbs v), f x = v x) :
        UniformSpace.comap (⇑f) inferInstance = PseudoMetricSpace.toUniformSpace

        If the absolute value v factors through an embedding f into a normed field, then the uniform structure associated to the absolute value is the same as the uniform structure induced by f.

        theorem WithAbs.isUniformInducing_of_comp {K : Type u_4} [Field K] {v : AbsoluteValue K } {L : Type u_5} [NormedField L] {f : WithAbs v →+* L} (h : ∀ (x : WithAbs v), f x = v x) :

        If the absolute value v factors through an embedding f into a normed field, then f is uniform inducing.

        @[reducible, inline]
        abbrev AbsoluteValue.completion {K : Type u_4} [Field K] (v : AbsoluteValue K ) :
        Type u_4

        The completion of a field with respect to a real absolute value.

        Equations
        Instances For
          @[reducible, inline]
          abbrev AbsoluteValue.Completion.extensionEmbedding_of_comp {K : Type u_4} [Field K] {v : AbsoluteValue K } {L : Type u_5} [NormedField L] [CompleteSpace L] {f : WithAbs v →+* L} (h : ∀ (x : WithAbs v), f x = v x) :
          v.completion →+* L

          If the absolute value of a normed field factors through an embedding into another normed field L, then we can extend that embedding to an embedding on the completion v.completion →+* L.

          Equations
          Instances For

            If the absolute value of a normed field factors through an embedding into another normed field, then the extended embedding v.completion →+* L preserves distances.

            If the absolute value of a normed field factors through an embedding into another normed field, then the extended embedding v.completion →+* L is an isometry.

            If the absolute value of a normed field factors through an embedding into another normed field, then the extended embedding v.completion →+* L is a closed embedding.

            theorem AbsoluteValue.Completion.locallyCompactSpace {K : Type u_4} [Field K] {v : AbsoluteValue K } {L : Type u_5} [NormedField L] [CompleteSpace L] {f : WithAbs v →+* L} [LocallyCompactSpace L] (h : ∀ (x : WithAbs v), f x = v x) :
            LocallyCompactSpace v.completion

            If the absolute value of a normed field factors through an embedding into another normed field that is locally compact, then the completion of the first normed field is also locally compact.