Ordered cancellative monoids #
Addition is monotone in an ordered cancellative additive commutative monoid.
Additive cancellation is compatible with the order in an ordered cancellative additive commutative monoid.
An ordered cancellative additive commutative monoid is an additive commutative monoid with a partial order, in which addition is cancellative and monotone.
Instances
Multiplication is monotone in an ordered cancellative commutative monoid.
Cancellation is compatible with the order in an ordered cancellative commutative monoid.
An ordered cancellative commutative monoid is a commutative monoid with a partial order, in which multiplication is cancellative and monotone.
Instances
Equations
- (_ : ContravariantClass α α (fun x x_1 => x + x_1) fun x x_1 => x ≤ x_1) = (_ : ContravariantClass α α (fun x x_1 => x + x_1) fun x x_1 => x ≤ x_1)
Equations
- (_ : ContravariantClass M M (fun x x_1 => x + x_1) fun x x_1 => x < x_1) = (_ : ContravariantClass M M (fun x x_1 => x + x_1) fun x x_1 => x < x_1)
Equations
- (_ : ContravariantClass M M (Function.swap fun x x_1 => x + x_1) fun x x_1 => x < x_1) = (_ : ContravariantClass M M (Function.swap fun x x_1 => x + x_1) fun x x_1 => x < x_1)
Equations
- (_ : ∀ (x : α), AddMonoid.nsmul 0 x = 0) = (_ : ∀ (x : α), AddMonoid.nsmul 0 x = 0)
Equations
- (_ : ∀ (n : ℕ) (x : α), AddMonoid.nsmul (n + 1) x = x + AddMonoid.nsmul n x) = (_ : ∀ (n : ℕ) (x : α), AddMonoid.nsmul (n + 1) x = x + AddMonoid.nsmul n x)
Equations
- OrderedCancelAddCommMonoid.toCancelAddCommMonoid = let src := inst; AddCancelCommMonoid.mk (_ : ∀ (a b : α), a + b = b + a)
Equations
- OrderedCancelCommMonoid.toCancelCommMonoid = let src := inst; CancelCommMonoid.mk (_ : ∀ (a b : α), a * b = b * a)
A linear order is total.
In a linearly ordered type, we assume the order relations are all decidable.
decidable_le : DecidableRel fun x x_1 => x ≤ x_1In a linearly ordered type, we assume the order relations are all decidable.
decidable_eq : DecidableEq αIn a linearly ordered type, we assume the order relations are all decidable.
decidable_lt : DecidableRel fun x x_1 => x < x_1The minimum function is equivalent to the one you get from
minOfLe
.The minimum function is equivalent to the one you get from
maxOfLe
.
A linearly ordered cancellative additive commutative monoid is an additive commutative monoid with a decidable linear order in which addition is cancellative and monotone.
Instances
A linear order is total.
In a linearly ordered type, we assume the order relations are all decidable.
decidable_le : DecidableRel fun x x_1 => x ≤ x_1In a linearly ordered type, we assume the order relations are all decidable.
decidable_eq : DecidableEq αIn a linearly ordered type, we assume the order relations are all decidable.
decidable_lt : DecidableRel fun x x_1 => x < x_1The minimum function is equivalent to the one you get from
minOfLe
.The minimum function is equivalent to the one you get from
maxOfLe
.
A linearly ordered cancellative commutative monoid is a commutative monoid with a linear order in which multiplication is cancellative and monotone.