Documentation

Mathlib.Analysis.Normed.Order.Basic

Ordered normed spaces #

In this file, we define classes for fields and groups that are both normed and ordered. These are mostly useful to avoid diamonds during type class inference.

A NormedOrderedAddGroup is an additive group that is both a NormedAddCommGroup and an OrderedAddCommGroup. This class is necessary to avoid diamonds caused by both classes carrying their own group structure.

Instances
    class NormedOrderedGroup (α : Type u_2) extends OrderedCommGroup , Norm , MetricSpace :
    Type u_2

    A NormedOrderedGroup is a group that is both a NormedCommGroup and an OrderedCommGroup. This class is necessary to avoid diamonds caused by both classes carrying their own group structure.

    Instances

      A NormedLinearOrderedAddGroup is an additive group that is both a NormedAddCommGroup and a LinearOrderedAddCommGroup. This class is necessary to avoid diamonds caused by both classes carrying their own group structure.

      Instances

        A NormedLinearOrderedGroup is a group that is both a NormedCommGroup and a LinearOrderedCommGroup. This class is necessary to avoid diamonds caused by both classes carrying their own group structure.

        Instances

          A NormedLinearOrderedField is a field that is both a NormedField and a LinearOrderedField. This class is necessary to avoid diamonds.

          Instances
            Equations
            Equations
            Equations
            Equations
            Equations
            • OrderDual.normedOrderedAddGroup = let __src := NormedOrderedAddGroup.toNormedAddCommGroup; let __src_1 := OrderDual.orderedAddCommGroup; NormedOrderedAddGroup.mk
            theorem OrderDual.normedOrderedAddGroup.proof_1 {α : Type u_1} [NormedOrderedAddGroup α] (a : αᵒᵈ) (b : αᵒᵈ) :
            a b∀ (c : αᵒᵈ), c + a c + b
            Equations
            • OrderDual.normedOrderedGroup = let __src := NormedOrderedGroup.toNormedCommGroup; let __src_1 := OrderDual.orderedCommGroup; NormedOrderedGroup.mk
            theorem OrderDual.normedLinearOrderedAddGroup.proof_2 {α : Type u_1} [NormedLinearOrderedAddGroup α] (a : αᵒᵈ) (b : αᵒᵈ) :
            min a b = if a b then a else b
            Equations
            theorem OrderDual.normedLinearOrderedAddGroup.proof_3 {α : Type u_1} [NormedLinearOrderedAddGroup α] (a : αᵒᵈ) (b : αᵒᵈ) :
            max a b = if a b then b else a
            Equations
            Equations
            • Additive.normedOrderedAddGroup = let __src := Additive.normedAddCommGroup; let __src_1 := Additive.orderedAddCommGroup; NormedOrderedAddGroup.mk
            Equations
            • Multiplicative.normedOrderedGroup = let __src := Multiplicative.normedCommGroup; let __src_1 := Multiplicative.orderedCommGroup; NormedOrderedGroup.mk
            Equations
            • Additive.normedLinearOrderedAddGroup = let __src := Additive.normedAddCommGroup; let __src_1 := Additive.linearOrderedAddCommGroup; NormedLinearOrderedAddGroup.mk
            Equations
            • Multiplicative.normedlinearOrderedGroup = let __src := Multiplicative.normedCommGroup; let __src_1 := Multiplicative.linearOrderedCommGroup; NormedLinearOrderedGroup.mk