Documentation

Mathlib.Algebra.Order.GroupWithZero.Canonical

Linearly ordered commutative groups and monoids with a zero element adjoined #

This file sets up a special class of linearly ordered commutative monoids that show up as the target of so-called “valuations” in algebraic number theory.

Usually, in the informal literature, these objects are constructed by taking a linearly ordered commutative group Γ and formally adjoining a zero element: Γ ∪ {0}.

The disadvantage is that a type such as NNReal is not of that form, whereas it is a very common target for valuations. The solutions is to use a typeclass, and that is exactly what we do in this file.

A linearly ordered commutative monoid with a zero element.

Instances

    A linearly ordered commutative group with a zero element.

    Instances
      @[reducible, inline]
      abbrev Function.Injective.linearOrderedCommMonoidWithZero {α : Type u_1} [LinearOrderedCommMonoidWithZero α] {β : Type u_3} [Zero β] [Bot β] [One β] [Mul β] [Pow β ] [LE β] [LT β] [Max β] [Min β] [Ord β] [DecidableEq β] [DecidableLE β] [DecidableLT β] (f : βα) (hf : Injective f) (zero : f 0 = 0) (one : f 1 = 1) (mul : ∀ (x y : β), f (x * y) = f x * f y) (npow : ∀ (x : β) (n : ), f (x ^ n) = f x ^ n) (le : ∀ {x y : β}, f x f y x y) (lt : ∀ {x y : β}, f x < f y x < y) (hsup : ∀ (x y : β), f (xy) = max (f x) (f y)) (hinf : ∀ (x y : β), f (xy) = min (f x) (f y)) (bot : f = ) (compare : ∀ (x y : β), compare (f x) (f y) = compare x y) :

      Pullback a LinearOrderedCommMonoidWithZero under an injective map. See note [reducible non-instances].

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem zero_le' {α : Type u_1} [LinearOrderedCommMonoidWithZero α] {a : α} :
        0 a
        @[simp]
        theorem not_lt_zero' {α : Type u_1} [LinearOrderedCommMonoidWithZero α] {a : α} :
        ¬a < 0
        @[simp]
        theorem le_zero_iff {α : Type u_1} [LinearOrderedCommMonoidWithZero α] {a : α} :
        a 0 a = 0
        theorem zero_lt_iff {α : Type u_1} [LinearOrderedCommMonoidWithZero α] {a : α} :
        0 < a a 0
        theorem ne_zero_of_lt {α : Type u_1} [LinearOrderedCommMonoidWithZero α] {a b : α} (h : b < a) :
        a 0

        See also bot_eq_zero and bot_eq_zero' for canonically ordered monoids.

        Equations
        • One or more equations did not get rendered due to their size.
        Equations
        • One or more equations did not get rendered due to their size.
        theorem pow_pos_iff {α : Type u_1} [LinearOrderedCommMonoidWithZero α] {a : α} {n : } [NoZeroDivisors α] (hn : n 0) :
        0 < a ^ n 0 < a
        @[simp]
        theorem Units.zero_lt {α : Type u_1} [LinearOrderedCommGroupWithZero α] (u : αˣ) :
        0 < u
        theorem mul_inv_lt_of_lt_mul₀ {α : Type u_1} [LinearOrderedCommGroupWithZero α] {a b c : α} (h : a < b * c) :
        a * c⁻¹ < b
        theorem inv_mul_lt_of_lt_mul₀ {α : Type u_1} [LinearOrderedCommGroupWithZero α] {a b c : α} (h : a < b * c) :
        b⁻¹ * a < c
        theorem lt_of_mul_lt_mul_of_le₀ {α : Type u_1} [LinearOrderedCommGroupWithZero α] {a b c d : α} (h : a * b < c * d) (hc : 0 < c) (hh : c a) :
        b < d
        Equations
        • One or more equations did not get rendered due to their size.
        Equations
        • One or more equations did not get rendered due to their size.
        Equations
        • One or more equations did not get rendered due to their size.
        instance WithZero.instBot {α : Type u_1} :
        Equations
        theorem WithZero.zero_eq_bot {α : Type u_1} :
        0 =
        @[instance 10]
        instance WithZero.le {α : Type u_1} [LE α] :
        Equations
        theorem WithZero.le_def {α : Type u_1} [LE α] {x y : WithZero α} :
        x y ∀ (a : α), x = a (b : α), y = b a b
        @[simp]
        theorem WithZero.coe_le_coe {α : Type u_1} [LE α] {a b : α} :
        a b a b
        theorem WithZero.not_coe_le_zero {α : Type u_1} [LE α] (a : α) :
        ¬a 0
        @[simp]
        theorem WithZero.zero_le {α : Type u_1} [LE α] (a : WithZero α) :
        0 a
        @[simp]
        theorem WithZero.nonpos_iff_eq_zero {α : Type u_1} [LE α] {x : WithZero α} :
        x 0 x = 0

        There is a general version le_zero_iff, but this lemma does not require a PartialOrder.

        theorem WithZero.coe_le_iff {α : Type u_1} [LE α] {x : WithZero α} {a : α} :
        a x (b : α), x = b a b
        theorem WithZero.le_coe_iff {α : Type u_1} [LE α] {x : WithZero α} {b : α} :
        x b ∀ (a : α), x = aa b
        theorem IsMax.withZero {α : Type u_1} [LE α] {a : α} (h : IsMax a) :
        IsMax a
        theorem WithZero.le_unzero_iff {α : Type u_1} [LE α] {y : WithZero α} {a : α} (hy : y 0) :
        a unzero hy a y
        theorem WithZero.unbot_le_iff {α : Type u_1} [LE α] {x : WithZero α} {b : α} (hx : x 0) :
        unzero hx b x b
        @[simp]
        theorem WithZero.one_le_coe {α : Type u_1} [LE α] {a : α} [One α] :
        1 a 1 a
        @[simp]
        theorem WithZero.coe_le_one {α : Type u_1} [LE α] {a : α} [One α] :
        a 1 a 1
        @[simp]
        theorem WithZero.unzero_le_unzero {α : Type u_1} [LE α] {x y : WithZero α} (hx : x 0) (hy : y 0) :
        unzero hx unzero hy x y
        @[instance 10]
        instance WithZero.instLT {α : Type u_1} [LT α] :

        The order on WithZero α, defined by ⊥ < ↑a and a < b → ↑a < ↑b.

        Equations
        theorem WithZero.lt_def {α : Type u_1} [LT α] {x y : WithZero α} :
        x < y (b : α), y = b ∀ (a : α), x = aa < b
        @[simp]
        theorem WithZero.coe_lt_coe {α : Type u_1} [LT α] {a b : α} :
        a < b a < b
        @[simp]
        theorem WithZero.zero_lt_coe {α : Type u_1} [LT α] (a : α) :
        0 < a
        @[simp]
        theorem WithZero.not_lt_zero {α : Type u_1} [LT α] (a : WithZero α) :
        ¬a < 0
        theorem WithZero.lt_iff_exists_coe {α : Type u_1} [LT α] {x y : WithZero α} :
        x < y (b : α), y = b x < b
        theorem WithZero.lt_coe_iff {α : Type u_1} [LT α] {x : WithZero α} {b : α} :
        x < b ∀ (a : α), x = aa < b
        theorem WithZero.pos_iff_ne_zero {α : Type u_1} [LT α] {x : WithZero α} :
        0 < x x 0

        A version of pos_iff_ne_zero for WithZero that only requires LT α, not PartialOrder α.

        theorem WithZero.lt_unzero_iff {α : Type u_1} [LT α] {y : WithZero α} {a : α} (hy : y 0) :
        a < unzero hy a < y
        theorem WithZero.unzero_lt_iff {α : Type u_1} [LT α] {x : WithZero α} {b : α} (hx : x 0) :
        unzero hx < b x < b
        @[simp]
        theorem WithZero.one_lt_coe {α : Type u_1} [LT α] {a : α} [One α] :
        1 < a 1 < a
        @[simp]
        theorem WithZero.coe_lt_one {α : Type u_1} [LT α] {a : α} [One α] :
        a < 1 a < 1
        theorem WithZero.addLeftMono {α : Type u_1} [Preorder α] [AddZeroClass α] [AddLeftMono α] (h : ∀ (a : α), 0 a) :
        theorem WithZero.map'_mono {α : Type u_1} {β : Type u_2} [Preorder α] [Preorder β] [MulOneClass α] [MulOneClass β] {f : α →* β} (hf : Monotone f) :
        Monotone (map' f)
        theorem WithZero.map'_strictMono {α : Type u_1} {β : Type u_2} [Preorder α] [Preorder β] [MulOneClass α] [MulOneClass β] {f : α →* β} (hf : StrictMono f) :
        theorem WithZero.exists_ne_zero_and_lt {α : Type u_1} [Preorder α] {x : WithZero α} [NoMinOrder α] (hx : x 0) :
        (y : WithZero α), y 0 y < x
        theorem WithZero.toAdd_unzero_lt_of_lt_ofAdd {α : Type u_1} [Preorder α] {a : WithZero (Multiplicative α)} {b : α} (ha : a 0) (h : a < (Multiplicative.ofAdd b)) :
        theorem WithZero.lt_ofAdd_of_toAdd_unzero_lt {α : Type u_1} [Preorder α] {a : WithZero (Multiplicative α)} {b : α} (ha : a 0) (h : Multiplicative.toAdd (unzero ha) < b) :
        theorem WithZero.lt_ofAdd_iff {α : Type u_1} [Preorder α] {a : WithZero (Multiplicative α)} {b : α} (ha : a 0) :
        theorem WithZero.toAdd_unzero_le_of_lt_ofAdd {α : Type u_1} [Preorder α] {a : WithZero (Multiplicative α)} {b : α} (ha : a 0) (h : a (Multiplicative.ofAdd b)) :
        theorem WithZero.le_ofAdd_of_toAdd_unzero_le {α : Type u_1} [Preorder α] {a : WithZero (Multiplicative α)} {b : α} (ha : a 0) (h : Multiplicative.toAdd (unzero ha) b) :
        theorem WithZero.le_ofAdd_iff {α : Type u_1} [Preorder α] {a : WithZero (Multiplicative α)} {b : α} (ha : a 0) :
        Equations
        • One or more equations did not get rendered due to their size.
        theorem WithZero.coe_sup {α : Type u_1} [SemilatticeSup α] (a b : α) :
        (ab) = ab
        Equations
        theorem WithZero.coe_inf {α : Type u_1} [SemilatticeInf α] (a b : α) :
        (ab) = ab
        instance WithZero.instLattice {α : Type u_1} [Lattice α] :
        Equations
        instance WithZero.isTotal_le {α : Type u_1} [Preorder α] [IsTotal α fun (x1 x2 : α) => x1 x2] :
        IsTotal (WithZero α) fun (x1 x2 : WithZero α) => x1 x2
        theorem WithZero.le_max_iff {α : Type u_1} [LinearOrder α] {a b c : α} :
        a max b c a max b c
        theorem WithZero.min_le_iff {α : Type u_1} [LinearOrder α] {a b c : α} :
        min a b c min a b c
        theorem WithZero.exists_ne_zero_and_le_and_le {α : Type u_1} [LinearOrder α] {x y : WithZero α} (hx : x 0) (hy : y 0) :
        (z : WithZero α), z 0 z x z y
        theorem WithZero.exists_ne_zero_and_lt_and_lt {α : Type u_1} [LinearOrder α] {x y : WithZero α} [NoMinOrder α] (hx : x 0) (hy : y 0) :
        (z : WithZero α), z 0 z < x z < y
        theorem WithZero.isOrderedAddMonoid {α : Type u_1} [AddCommMonoid α] [PartialOrder α] [IsOrderedAddMonoid α] (zero_le : ∀ (a : α), 0 a) :

        If 0 is the least element in α, then WithZero α is an ordered AddMonoid.

        Adding a new zero to a canonically ordered additive monoid produces another one.

        Equations
        • One or more equations did not get rendered due to their size.
        Equations
        • One or more equations did not get rendered due to their size.

        Exponential and logarithm #

        @[simp]
        theorem WithZero.exp_le_exp {G : Type u_3} [Preorder G] {a b : G} :
        exp a exp b a b
        @[simp]
        theorem WithZero.exp_lt_exp {G : Type u_3} [Preorder G] {a b : G} :
        exp a < exp b a < b
        @[simp]
        theorem WithZero.exp_pos {G : Type u_3} [Preorder G] {a : G} :
        0 < exp a
        @[simp]
        theorem WithZero.log_le_log {G : Type u_3} [Preorder G] [AddGroup G] {x y : WithZero (Multiplicative G)} (hx : x 0) (hy : y 0) :
        x.log y.log x y
        @[simp]
        theorem WithZero.log_lt_log {G : Type u_3} [Preorder G] [AddGroup G] {x y : WithZero (Multiplicative G)} (hx : x 0) (hy : y 0) :
        x.log < y.log x < y
        theorem WithZero.log_le_iff_le_exp {G : Type u_3} [Preorder G] {a : G} [AddGroup G] {x : WithZero (Multiplicative G)} (hx : x 0) :
        x.log a x exp a
        theorem WithZero.log_lt_iff_lt_exp {G : Type u_3} [Preorder G] {a : G} [AddGroup G] {x : WithZero (Multiplicative G)} (hx : x 0) :
        x.log < a x < exp a
        theorem WithZero.le_log_iff_exp_le {G : Type u_3} [Preorder G] {a : G} [AddGroup G] {x : WithZero (Multiplicative G)} (hx : x 0) :
        a x.log exp a x
        theorem WithZero.lt_log_iff_exp_lt {G : Type u_3} [Preorder G] {a : G} [AddGroup G] {x : WithZero (Multiplicative G)} (hx : x 0) :
        a < x.log exp a < x
        theorem WithZero.le_exp_of_log_le {G : Type u_3} [Preorder G] {a : G} [AddGroup G] {x : WithZero (Multiplicative G)} (hxa : x.log a) :
        x exp a
        theorem WithZero.lt_exp_of_log_lt {G : Type u_3} [Preorder G] {a : G} [AddGroup G] {x : WithZero (Multiplicative G)} (hxa : x.log < a) :
        x < exp a
        theorem WithZero.le_log_of_exp_le {G : Type u_3} [Preorder G] {a : G} [AddGroup G] {x : WithZero (Multiplicative G)} (hax : exp a x) :
        a x.log
        theorem WithZero.lt_log_of_exp_lt {G : Type u_3} [Preorder G] {a : G} [AddGroup G] {x : WithZero (Multiplicative G)} (hax : exp a < x) :
        a < x.log

        The exponential map as an order isomorphism between G and Gᵐ⁰ˣ.

        Equations
        Instances For
          @[simp]
          theorem WithZero.val_inv_expOrderIso_apply {G : Type u_3} [Preorder G] [AddGroup G] (a✝ : G) :
          @[simp]
          theorem WithZero.val_expOrderIso_apply {G : Type u_3} [Preorder G] [AddGroup G] (a✝ : G) :
          (expOrderIso a✝) = (Multiplicative.ofAdd a✝)

          The logarithm as an order isomorphism between Gᵐ⁰ˣ and G.

          Equations
          Instances For
            @[simp]
            theorem WithZero.val_logOrderIso_symm_apply {G : Type u_3} [Preorder G] [AddGroup G] (a✝ : G) :
            theorem WithZero.lt_mul_exp_iff_le {x y : WithZero (Multiplicative )} (hy : y 0) :
            x < y * exp 1 x y