Documentation

Mathlib.Analysis.Normed.Field.Lemmas

Normed fields #

In this file we continue building the theory of normed division rings and fields.

Some useful results that relate the topology of the normed field to the discrete topology include:

def DilationEquiv.mulLeft {α : Type u_1} [NormedDivisionRing α] (a : α) (ha : a 0) :
α ≃ᵈ α

Multiplication by a nonzero element a on the left as a DilationEquiv of a normed division ring.

Equations
Instances For
    @[simp]
    theorem DilationEquiv.mulLeft_apply {α : Type u_1} [NormedDivisionRing α] (a : α) (ha : a 0) (x : α) :
    (mulLeft a ha) x = a * x
    @[simp]
    theorem DilationEquiv.mulLeft_symm_apply {α : Type u_1} [NormedDivisionRing α] (a : α) (ha : a 0) (x : α) :
    (mulLeft a ha).symm x = a⁻¹ * x
    def DilationEquiv.mulRight {α : Type u_1} [NormedDivisionRing α] (a : α) (ha : a 0) :
    α ≃ᵈ α

    Multiplication by a nonzero element a on the right as a DilationEquiv of a normed division ring.

    Equations
    Instances For
      @[simp]
      theorem DilationEquiv.mulRight_apply {α : Type u_1} [NormedDivisionRing α] (a : α) (ha : a 0) (x : α) :
      (mulRight a ha) x = x * a
      @[simp]
      theorem DilationEquiv.mulRight_symm_apply {α : Type u_1} [NormedDivisionRing α] (a : α) (ha : a 0) (x : α) :
      (mulRight a ha).symm x = x * a⁻¹
      @[simp]
      theorem Filter.map_mul_left_cobounded {α : Type u_1} [NormedDivisionRing α] {a : α} (ha : a 0) :
      map (fun (x : α) => a * x) (Bornology.cobounded α) = Bornology.cobounded α
      @[simp]
      theorem Filter.map_mul_right_cobounded {α : Type u_1} [NormedDivisionRing α] {a : α} (ha : a 0) :
      map (fun (x : α) => x * a) (Bornology.cobounded α) = Bornology.cobounded α
      theorem Filter.tendsto_mul_left_cobounded {α : Type u_1} [NormedDivisionRing α] {a : α} (ha : a 0) :
      Tendsto (fun (x : α) => a * x) (Bornology.cobounded α) (Bornology.cobounded α)

      Multiplication on the left by a nonzero element of a normed division ring tends to infinity at infinity.

      theorem Filter.tendsto_mul_right_cobounded {α : Type u_1} [NormedDivisionRing α] {a : α} (ha : a 0) :
      Tendsto (fun (x : α) => x * a) (Bornology.cobounded α) (Bornology.cobounded α)

      Multiplication on the right by a nonzero element of a normed division ring tends to infinity at infinity.

      @[instance 100]

      A normed division ring is a topological division ring.

      @[deprecated NormedDivisionRing.to_isTopologicalDivisionRing (since := "2025-03-25")]

      Alias of NormedDivisionRing.to_isTopologicalDivisionRing.


      A normed division ring is a topological division ring.

      @[deprecated NormedField.tendsto_norm_inv_nhdsNE_zero_atTop (since := "2024-12-22")]

      Alias of NormedField.tendsto_norm_inv_nhdsNE_zero_atTop.

      @[deprecated NormedField.tendsto_norm_zpow_nhdsNE_zero_atTop (since := "2024-12-22")]

      Alias of NormedField.tendsto_norm_zpow_nhdsNE_zero_atTop.

      A normed field is either nontrivially normed or has a discrete topology. In the discrete topology case, all the norms are 1, by norm_eq_one_iff_ne_zero_of_discrete. The nontrivially normed field instance is provided by a subtype with a proof that the forgetful inheritance to the existing NormedField instance is definitionally true. This allows one to have the new NontriviallyNormedField instance without data clashes.

      @[simp]
      theorem NormedField.continuousAt_zpow {𝕜 : Type u_4} [NontriviallyNormedField 𝕜] {n : } {x : 𝕜} :
      ContinuousAt (fun (x : 𝕜) => x ^ n) x x 0 0 n
      @[simp]