Documentation

Mathlib.Analysis.Normed.Ring.Seminorm

Seminorms and norms on rings #

This file defines seminorms and norms on rings. These definitions are useful when one needs to consider multiple (semi)norms on a given ring.

Main declarations #

For a ring R:

Notes #

The corresponding hom classes are defined in Mathlib.Analysis.Order.Hom.Basic to be used by absolute values.

References #

Tags #

ring_seminorm, ring_norm

structure RingSeminorm (R : Type u_4) [NonUnitalNonAssocRing R] extends AddGroupSeminorm :
Type u_4

A seminorm on a ring R is a function f : R → ℝ that preserves zero, takes nonnegative values, is subadditive and submultiplicative and such that f (-x) = f x for all x ∈ R.

  • toFun : R
  • map_zero' : self.toFun 0 = 0
  • add_le' : ∀ (r s : R), self.toFun (r + s) self.toFun r + self.toFun s
  • neg' : ∀ (r : R), self.toFun (-r) = self.toFun r
  • mul_le' : ∀ (x y : R), self.toFun (x * y) self.toFun x * self.toFun y

    The property of a RingSeminorm that for all x and y in the ring, the norm of x * y is less than the norm of x times the norm of y.

Instances For
    structure RingNorm (R : Type u_4) [NonUnitalNonAssocRing R] extends RingSeminorm :
    Type u_4

    A function f : R → ℝ is a norm on a (nonunital) ring if it is a seminorm and f x = 0 implies x = 0.

    • toFun : R
    • map_zero' : self.toFun 0 = 0
    • add_le' : ∀ (r s : R), self.toFun (r + s) self.toFun r + self.toFun s
    • neg' : ∀ (r : R), self.toFun (-r) = self.toFun r
    • mul_le' : ∀ (x y : R), self.toFun (x * y) self.toFun x * self.toFun y
    • eq_zero_of_map_eq_zero' : ∀ (x : R), self.toFun x = 0x = 0

      If the image under the seminorm is zero, then the argument is zero.

    Instances For
      structure MulRingSeminorm (R : Type u_4) [NonAssocRing R] extends AddGroupSeminorm :
      Type u_4

      A multiplicative seminorm on a ring R is a function f : R → ℝ that preserves zero and multiplication, takes nonnegative values, is subadditive and such that f (-x) = f x for all x.

      • toFun : R
      • map_zero' : self.toFun 0 = 0
      • add_le' : ∀ (r s : R), self.toFun (r + s) self.toFun r + self.toFun s
      • neg' : ∀ (r : R), self.toFun (-r) = self.toFun r
      • map_one' : self.toFun 1 = 1

        The proposition that the function preserves 1

      • map_mul' : ∀ (x y : R), self.toFun (x * y) = self.toFun x * self.toFun y

        The proposition that the function preserves multiplication

      Instances For
        structure MulRingNorm (R : Type u_4) [NonAssocRing R] extends MulRingSeminorm :
        Type u_4

        A multiplicative norm on a ring R is a multiplicative ring seminorm such that f x = 0 implies x = 0.

        • toFun : R
        • map_zero' : self.toFun 0 = 0
        • add_le' : ∀ (r s : R), self.toFun (r + s) self.toFun r + self.toFun s
        • neg' : ∀ (r : R), self.toFun (-r) = self.toFun r
        • map_one' : self.toFun 1 = 1
        • map_mul' : ∀ (x y : R), self.toFun (x * y) = self.toFun x * self.toFun y
        • eq_zero_of_map_eq_zero' : ∀ (x : R), self.toFun x = 0x = 0

          If the image under the seminorm is zero, then the argument is zero.

        Instances For
          Equations
          • RingSeminorm.funLike = { coe := fun (f : RingSeminorm R) => f.toFun, coe_injective' := }
          @[simp]
          theorem RingSeminorm.toFun_eq_coe {R : Type u_2} [NonUnitalRing R] (p : RingSeminorm R) :
          p.toAddGroupSeminorm = p
          theorem RingSeminorm.ext {R : Type u_2} [NonUnitalRing R] {p : RingSeminorm R} {q : RingSeminorm R} :
          (∀ (x : R), p x = q x)p = q
          Equations
          • RingSeminorm.instZeroRingSeminormToNonUnitalNonAssocRing = { zero := let __src := Zero.zero; { toAddGroupSeminorm := __src, mul_le' := } }
          theorem RingSeminorm.eq_zero_iff {R : Type u_2} [NonUnitalRing R] {p : RingSeminorm R} :
          p = 0 ∀ (x : R), p x = 0
          theorem RingSeminorm.ne_zero_iff {R : Type u_2} [NonUnitalRing R] {p : RingSeminorm R} :
          p 0 ∃ (x : R), p x 0
          Equations
          • RingSeminorm.instInhabitedRingSeminormToNonUnitalNonAssocRing = { default := 0 }

          The trivial seminorm on a ring R is the RingSeminorm taking value 0 at 0 and 1 at every other element.

          Equations
          • RingSeminorm.instOneRingSeminormToNonUnitalNonAssocRing = { one := let __src := 1; { toAddGroupSeminorm := __src, mul_le' := } }
          @[simp]
          theorem RingSeminorm.apply_one {R : Type u_2} [NonUnitalRing R] [DecidableEq R] (x : R) :
          1 x = if x = 0 then 0 else 1
          theorem RingSeminorm.seminorm_one_eq_one_iff_ne_zero {R : Type u_2} [Ring R] (p : RingSeminorm R) (hp : p 1 1) :
          p 1 = 1 p 0

          The norm of a NonUnitalSeminormedRing as a RingSeminorm.

          Equations
          Instances For
            instance RingNorm.funLike {R : Type u_2} [NonUnitalRing R] :
            Equations
            • RingNorm.funLike = { coe := fun (f : RingNorm R) => f.toFun, coe_injective' := }
            Equations
            • =
            theorem RingNorm.toFun_eq_coe {R : Type u_2} [NonUnitalRing R] (p : RingNorm R) :
            p.toFun = p
            theorem RingNorm.ext {R : Type u_2} [NonUnitalRing R] {p : RingNorm R} {q : RingNorm R} :
            (∀ (x : R), p x = q x)p = q

            The trivial norm on a ring R is the RingNorm taking value 0 at 0 and 1 at every other element.

            Equations
            @[simp]
            theorem RingNorm.apply_one (R : Type u_2) [NonUnitalRing R] [DecidableEq R] (x : R) :
            1 x = if x = 0 then 0 else 1
            Equations
            • MulRingSeminorm.funLike = { coe := fun (f : MulRingSeminorm R) => f.toFun, coe_injective' := }
            @[simp]
            theorem MulRingSeminorm.toFun_eq_coe {R : Type u_2} [NonAssocRing R] (p : MulRingSeminorm R) :
            p.toAddGroupSeminorm = p
            theorem MulRingSeminorm.ext {R : Type u_2} [NonAssocRing R] {p : MulRingSeminorm R} {q : MulRingSeminorm R} :
            (∀ (x : R), p x = q x)p = q

            The trivial seminorm on a ring R is the MulRingSeminorm taking value 0 at 0 and 1 at every other element.

            Equations
            • MulRingSeminorm.instOneMulRingSeminorm = { one := let __src := 1; { toAddGroupSeminorm := __src, map_one' := , map_mul' := } }
            @[simp]
            theorem MulRingSeminorm.apply_one {R : Type u_2} [NonAssocRing R] [DecidableEq R] [NoZeroDivisors R] [Nontrivial R] (x : R) :
            1 x = if x = 0 then 0 else 1
            Equations
            • MulRingSeminorm.instInhabitedMulRingSeminorm = { default := 1 }
            Equations
            • MulRingNorm.funLike = { coe := fun (f : MulRingNorm R) => f.toFun, coe_injective' := }
            theorem MulRingNorm.toFun_eq_coe {R : Type u_2} [NonAssocRing R] (p : MulRingNorm R) :
            p.toFun = p
            theorem MulRingNorm.ext {R : Type u_2} [NonAssocRing R] {p : MulRingNorm R} {q : MulRingNorm R} :
            (∀ (x : R), p x = q x)p = q

            The trivial norm on a ring R is the MulRingNorm taking value 0 at 0 and 1 at every other element.

            Equations
            @[simp]
            theorem MulRingNorm.apply_one (R : Type u_2) [NonAssocRing R] [DecidableEq R] [NoZeroDivisors R] [Nontrivial R] (x : R) :
            1 x = if x = 0 then 0 else 1
            def MulRingNorm.equiv {R : Type u_4} [Ring R] (f : MulRingNorm R) (g : MulRingNorm R) :

            Two multiplicative ring norms f, g on R are equivalent if there exists a positive constant c such that for all x ∈ R, (f x)^c = g x.

            Equations
            Instances For
              theorem MulRingNorm.equiv_refl {R : Type u_4} [Ring R] (f : MulRingNorm R) :

              Equivalence of multiplicative ring norms is reflexive.

              theorem MulRingNorm.equiv_symm {R : Type u_4} [Ring R] {f : MulRingNorm R} {g : MulRingNorm R} (hfg : MulRingNorm.equiv f g) :

              Equivalence of multiplicative ring norms is symmetric.

              theorem MulRingNorm.equiv_trans {R : Type u_4} [Ring R] {f : MulRingNorm R} {g : MulRingNorm R} {k : MulRingNorm R} (hfg : MulRingNorm.equiv f g) (hgk : MulRingNorm.equiv g k) :

              Equivalence of multiplicative ring norms is transitive.

              def RingSeminorm.toRingNorm {K : Type u_4} [Field K] (f : RingSeminorm K) (hnt : f 0) :

              A nonzero ring seminorm on a field K is a ring norm.

              Equations
              Instances For
                @[simp]
                theorem normRingNorm_toFun (R : Type u_4) [NonUnitalNormedRing R] :
                ∀ (a : R), (normRingNorm R).toFun a = a

                The norm of a NonUnitalNormedRing as a RingNorm.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  theorem MulRingNorm_nat_le_nat {R : Type u_4} [Ring R] (n : ) (f : MulRingNorm R) :
                  f n n

                  A multiplicative ring norm satisfies f n ≤ n for every n : ℕ.