Skip to content

Commit

Permalink
chore: fix a few docstrings (#1291)
Browse files Browse the repository at this point in the history
Fix a few docstrings still using the mathlib3 naming convention -- hard to notice these things while porting, but easy to notice when clicking round the docs.
  • Loading branch information
hrmacbeth committed Jan 2, 2023
1 parent bd48694 commit 24f600f
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 8 deletions.
8 changes: 4 additions & 4 deletions Mathlib/Algebra/Associated.lean
Expand Up @@ -373,7 +373,7 @@ theorem pow_not_prime {n : ℕ} (hn : n ≠ 1) : ¬Prime (a ^ n) := fun hp =>

end CancelCommMonoidWithZero

/-- Two elements of a `monoid` are `associated` if one of them is another one
/-- Two elements of a `Monoid` are `Associated` if one of them is another one
multiplied by a unit on the right. -/
def Associated [Monoid α] (x y : α) : Prop :=
∃ u : αˣ, x * u = y
Expand Down Expand Up @@ -730,9 +730,9 @@ theorem eq_of_prime_pow_eq' (hp₁ : Prime p₁) (hp₂ : Prime p₂) (hk₁ : 0

end UniqueUnits₀

/-- The quotient of a monoid by the `associated` relation. Two elements `x` and `y`
/-- The quotient of a monoid by the `Associated` relation. Two elements `x` and `y`
are associated iff there is a unit `u` such that `x * u = y`. There is a natural
monoid structure on `associates α`. -/
monoid structure on `Associates α`. -/
abbrev Associates (α : Type _) [Monoid α] : Type _ :=
Quotient (Associated.setoid α)
#align associates Associates
Expand All @@ -741,7 +741,7 @@ namespace Associates

open Associated

/-- The canonical quotient map from a monoid `α` into the `associates` of `α` -/
/-- The canonical quotient map from a monoid `α` into the `Associates` of `α` -/
protected abbrev mk {α : Type _} [Monoid α] (a : α) : Associates α :=
⟦a⟧
#align associates.mk Associates.mk
Expand Down
8 changes: 4 additions & 4 deletions Mathlib/Algebra/Order/Monoid/Basic.lean
Expand Up @@ -56,21 +56,21 @@ def Function.Injective.linearOrderedCommMonoid [LinearOrderedCommMonoid α] {β

-- TODO find a better home for the next two constructions.
/-- The order embedding sending `b` to `a * b`, for some fixed `a`.
See also `OrderIso.mul_left` when working in an ordered group. -/
See also `OrderIso.mulLeft` when working in an ordered group. -/
@[to_additive
"The order embedding sending `b` to `a + b`, for some fixed `a`.
See also `OrderIso.add_left` when working in an additive ordered group.",
See also `OrderIso.addLeft` when working in an additive ordered group.",
simps]
def OrderEmbedding.mulLeft {α : Type _} [Mul α] [LinearOrder α]
[CovariantClass α α (· * ·) (· < ·)] (m : α) : α ↪o α :=
OrderEmbedding.ofStrictMono (fun n => m * n) fun _ _ w => mul_lt_mul_left' w m
#align order_embedding.mul_left OrderEmbedding.mulLeft

/-- The order embedding sending `b` to `b * a`, for some fixed `a`.
See also `OrderIso.mul_right` when working in an ordered group. -/
See also `OrderIso.mulRight` when working in an ordered group. -/
@[to_additive
"The order embedding sending `b` to `b + a`, for some fixed `a`.
See also `OrderIso.add_right` when working in an additive ordered group.",
See also `OrderIso.addRight` when working in an additive ordered group.",
simps]
def OrderEmbedding.mulRight {α : Type _} [Mul α] [LinearOrder α]
[CovariantClass α α (swap (· * ·)) (· < ·)] (m : α) : α ↪o α :=
Expand Down

0 comments on commit 24f600f

Please sign in to comment.