Skip to content

Commit

Permalink
chore(Algebra/Order/Monoid/Prod): unify type names (#8273)
Browse files Browse the repository at this point in the history
Co-authored-by: madvorak <dvorakmartinbridge@seznam.cz>
  • Loading branch information
madvorak and madvorak committed Nov 8, 2023
1 parent 83bf88a commit 2f574a6
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions Mathlib/Algebra/Order/Monoid/Prod.lean
Expand Up @@ -14,16 +14,16 @@ import Mathlib.Data.Prod.Lex

namespace Prod

variable {α β M N : Type*}
variable {α β : Type*}

@[to_additive]
instance [OrderedCommMonoid α] [OrderedCommMonoid β] : OrderedCommMonoid (α × β) where
mul_le_mul_left _ _ h _ := ⟨mul_le_mul_left' h.1 _, mul_le_mul_left' h.2 _⟩

@[to_additive]
instance instOrderedCancelCommMonoid [OrderedCancelCommMonoid M] [OrderedCancelCommMonoid N] :
OrderedCancelCommMonoid (M × N) :=
{ (inferInstance : OrderedCommMonoid (M × N)) with
instance instOrderedCancelCommMonoid [OrderedCancelCommMonoid α] [OrderedCancelCommMonoid β] :
OrderedCancelCommMonoid (α × β) :=
{ (inferInstance : OrderedCommMonoid (α × β)) with
le_of_mul_le_mul_left :=
fun _ _ _ h ↦ ⟨le_of_mul_le_mul_left' h.1, le_of_mul_le_mul_left' h.2⟩ }

Expand Down

0 comments on commit 2f574a6

Please sign in to comment.