Documentation

Mathlib.Algebra.Order.Ring.Defs

Ordered rings and semirings #

This file develops the basics of ordered (semi)rings.

Each typeclass here comprises

For short,

Typeclasses #

Hierarchy #

The hardest part of proving order lemmas might be to figure out the correct generality and its corresponding typeclass. Here's an attempt at demystifying it. For each typeclass, we list its immediate predecessors and what conditions are added to each of them.

class IsOrderedRing (α : Type u_1) [Semiring α] [PartialOrder α] extends IsOrderedAddMonoid α, ZeroLEOneClass α :

An ordered semiring is a semiring with a partial order such that addition is monotone and multiplication by a nonnegative number is monotone.

  • add_le_add_left (a b : α) : a b∀ (c : α), c + a c + b
  • add_le_add_right (a b : α) : a b∀ (c : α), a + c b + c
  • mul_le_mul_of_nonneg_left (a b c : α) : a b0 cc * a c * b

    In an ordered semiring, we can multiply an inequality a ≤ b on the left by a non-negative element 0 ≤ c to obtain c * a ≤ c * b.

  • mul_le_mul_of_nonneg_right (a b c : α) : a b0 ca * c b * c

    In an ordered semiring, we can multiply an inequality a ≤ b on the right by a non-negative element 0 ≤ c to obtain a * c ≤ b * c.

Instances

    A strict ordered semiring is a nontrivial semiring with a partial order such that addition is strictly monotone and multiplication by a positive number is strictly monotone.

    Instances
      theorem IsOrderedRing.of_mul_nonneg {α : Type u} [Ring α] [PartialOrder α] [IsOrderedAddMonoid α] [ZeroLEOneClass α] (mul_nonneg : ∀ (a b : α), 0 a0 b0 a * b) :
      theorem IsStrictOrderedRing.of_mul_pos {α : Type u} [Ring α] [PartialOrder α] [IsOrderedAddMonoid α] [ZeroLEOneClass α] [Nontrivial α] (mul_pos : ∀ (a b : α), 0 < a0 < b0 < a * b) :
      @[instance 200]
      @[instance 200]

      Turn an ordered domain into a strict ordered ring.

      @[instance 100]

      Note that OrderDual does not satisfy any of the ordered ring typeclasses due to the zero_le_one field.

      class OrderedSemiring (α : Type u) extends Semiring α, OrderedAddCommMonoid α :

      An OrderedSemiring is a semiring with a partial order such that addition is monotone and multiplication by a nonnegative number is monotone.

      Instances
        class OrderedCommSemiring (α : Type u) extends OrderedSemiring α, CommSemiring α :

        An OrderedCommSemiring is a commutative semiring with a partial order such that addition is monotone and multiplication by a nonnegative number is monotone.

        Instances
          class OrderedRing (α : Type u) extends Ring α, OrderedAddCommGroup α :

          An OrderedRing is a ring with a partial order such that addition is monotone and multiplication by a nonnegative number is monotone.

          Instances
            class OrderedCommRing (α : Type u) extends OrderedRing α, CommRing α :

            An OrderedCommRing is a commutative ring with a partial order such that addition is monotone and multiplication by a nonnegative number is monotone.

            Instances

              A StrictOrderedSemiring is a nontrivial semiring with a partial order such that addition is strictly monotone and multiplication by a positive number is strictly monotone.

              Instances

                A StrictOrderedCommSemiring is a commutative semiring with a partial order such that addition is strictly monotone and multiplication by a positive number is strictly monotone.

                Instances
                  class StrictOrderedRing (α : Type u) extends Ring α, OrderedAddCommGroup α, Nontrivial α :

                  A StrictOrderedRing is a ring with a partial order such that addition is strictly monotone and multiplication by a positive number is strictly monotone.

                  Instances
                    class StrictOrderedCommRing (α : Type u_1) extends StrictOrderedRing α, CommRing α :
                    Type u_1

                    A StrictOrderedCommRing is a commutative ring with a partial order such that addition is strictly monotone and multiplication by a positive number is strictly monotone.

                    Instances

                      A LinearOrderedSemiring is a nontrivial semiring with a linear order such that addition is monotone and multiplication by a positive number is strictly monotone.

                      Instances

                        A LinearOrderedCommSemiring is a nontrivial commutative semiring with a linear order such that addition is monotone and multiplication by a positive number is strictly monotone.

                        Instances
                          class LinearOrderedRing (α : Type u) extends StrictOrderedRing α, LinearOrder α :

                          A LinearOrderedRing is a ring with a linear order such that addition is monotone and multiplication by a positive number is strictly monotone.

                          Instances

                            A LinearOrderedCommRing is a commutative ring with a linear order such that addition is monotone and multiplication by a positive number is strictly monotone.

                            Instances
                              @[instance 100]
                              Equations
                              • One or more equations did not get rendered due to their size.
                              theorem one_add_le_one_sub_mul_one_add {α : Type u} [OrderedRing α] {a b c : α} (h : a + b + b * c c) :
                              1 + a (1 - b) * (1 + c)
                              theorem one_add_le_one_add_mul_one_sub {α : Type u} [OrderedRing α] {a b c : α} (h : a + c + b * c b) :
                              1 + a (1 + b) * (1 - c)
                              theorem one_sub_le_one_sub_mul_one_add {α : Type u} [OrderedRing α] {a b c : α} (h : b + b * c a + c) :
                              1 - a (1 - b) * (1 + c)
                              theorem one_sub_le_one_add_mul_one_sub {α : Type u} [OrderedRing α] {a b c : α} (h : c + b * c a + b) :
                              1 - a (1 + b) * (1 - c)
                              @[instance 100]
                              Equations
                              @[reducible, inline]

                              A choice-free version of StrictOrderedSemiring.toOrderedSemiring to avoid using choice in basic Nat lemmas.

                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For
                                @[instance 100]
                                Equations
                                • One or more equations did not get rendered due to their size.
                                @[reducible, inline]

                                A choice-free version of StrictOrderedCommSemiring.toOrderedCommSemiring' to avoid using choice in basic Nat lemmas.

                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For
                                  @[instance 100]
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  @[instance 100]
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  @[reducible, inline]

                                  A choice-free version of StrictOrderedRing.toOrderedRing to avoid using choice in basic Int lemmas.

                                  Equations
                                  Instances For
                                    @[instance 100]
                                    Equations
                                    @[reducible, inline]

                                    A choice-free version of StrictOrderedCommRing.toOrderedCommRing to avoid using choice in basic Int lemmas.

                                    Equations
                                    • One or more equations did not get rendered due to their size.
                                    Instances For
                                      @[instance 100]
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      @[instance 100]
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      @[instance 100]
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      @[instance 100]
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      @[instance 100]
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      @[instance 100]
                                      Equations
                                      • One or more equations did not get rendered due to their size.