Documentation

Mathlib.Algebra.Order.Monoid.Submonoid

Ordered instances on submonoids #

A submonoid of an OrderedCommMonoid is an OrderedCommMonoid.

Equations

The submonoid of elements that are at least 1.

Equations
Instances For

    The submonoid of nonnegative elements.

    Equations
    Instances For
      @[simp]
      theorem Submonoid.coe_oneLE (M : Type u_1) [Monoid M] [Preorder M] [MulLeftMono M] :
      (oneLE M) = Set.Ici 1
      @[simp]
      theorem AddSubmonoid.coe_nonneg (M : Type u_1) [AddMonoid M] [Preorder M] [AddLeftMono M] :
      (nonneg M) = Set.Ici 0
      @[simp]
      theorem Submonoid.mem_oneLE {M : Type u_1} [Monoid M] [Preorder M] [MulLeftMono M] {a : M} :
      a oneLE M 1 a
      @[simp]
      theorem AddSubmonoid.mem_nonneg {M : Type u_1} [AddMonoid M] [Preorder M] [AddLeftMono M] {a : M} :
      a nonneg M 0 a