Zulip Chat Archive

Stream: maths

Topic: OrderedAddMonoid


Martin Dvořák (Oct 21 2023 at 13:28):

We have OrderedAddCommMonoid which is certainly meaningful.

import Mathlib.Algebra.Order.Monoid.Lemmas
import Mathlib.Order.BoundedOrder

class OrderedAddCommMonoid (α : Type*) extends AddCommMonoid α, PartialOrder α where
  /-- Addition is monotone in an `OrderedAddCommMonoid`. -/
  protected add_le_add_left :  a b : α, a  b   c : α, c + a  c + b

Would the following class make any (mathematical) sense?

import Mathlib.Algebra.Order.Monoid.Lemmas
import Mathlib.Order.BoundedOrder

class OrderedAddMonoid (α : Type*) extends AddMonoid α, PartialOrder α where
  protected add_le_add_left :  a b : α, a  b   c : α, c + a  c + b
  protected add_le_add_right :  a b : α, a  b   c : α, a + c  b + c

Martin Dvořák (Oct 21 2023 at 13:33):

Or OrderedMonoid rather.

Yaël Dillies (Oct 21 2023 at 13:36):

What's your use case?

Yaël Dillies (Oct 21 2023 at 13:37):

They are certainly people who study non-commutative orders, but those are pretty niche and we won't support them until they show up here.

Martin Dvořák (Oct 21 2023 at 13:41):

I don't have a use case, but I was thinking about lexicographical orderings on lists of ordered things.

Martin Dvořák (Oct 21 2023 at 13:42):

Actually no:

[1] < [1, 2]
[1, 3] > [1, 2, 3]

Yaël Dillies (Oct 21 2023 at 13:42):

Non-commutative orders do exist but they are pretty niche.

Jireh Loreaux (Oct 21 2023 at 15:28):

And the best ones involve star :laughing:

Frédéric Dupuis (Oct 21 2023 at 15:36):

Even then, addition is still commutative!

Antoine Chambert-Loir (Oct 21 2023 at 18:03):

Yaël Dillies said:

Non-commutative orders do exist but they are pretty niche.

In case of groups, they're not niche at all. For instance, the orderability of the braid group is an important theorem.

Yuyang Zhao (Oct 22 2023 at 21:06):

docs#Ordinal is an example.


Last updated: Dec 20 2023 at 11:08 UTC