Skip to content

Commit 5f2c0b7

Browse files
chore: tidy various files (#5268)
1 parent 0c4c62b commit 5f2c0b7

File tree

14 files changed

+122
-107
lines changed

14 files changed

+122
-107
lines changed

Diff for: Mathlib/Algebra/Category/Mon/FilteredColimits.lean

+9-10
Original file line numberDiff line numberDiff line change
@@ -37,15 +37,14 @@ open CategoryTheory
3737

3838
open CategoryTheory.Limits
3939

40-
open CategoryTheory.IsFiltered renaming max → max'
40+
open CategoryTheory.IsFiltered renaming max → max' -- avoid name collision with `_root_.max`.
4141

42-
-- avoid name collision with `_root_.max`.
4342
namespace MonCat.FilteredColimits
4443

4544
section
4645

47-
-- We use parameters here, mainly so we can have the abbreviations `M` and `M.mk` below, without
48-
-- passing around `F` all the time.
46+
-- Porting note: mathlib 3 used `parameters` here, mainly so we can have the abbreviations `M` and
47+
-- `M.mk` below, without passing around `F` all the time.
4948
variable {J : Type v} [SmallCategory J] (F : J ⥤ MonCat.{max v u})
5049

5150
/-- The colimit of `F ⋙ forget Mon` in the category of types.
@@ -114,13 +113,13 @@ set_option linter.uppercaseLean3 false in
114113
#align AddMon.filtered_colimits.colimit_zero_eq AddMonCat.FilteredColimits.colimit_zero_eq
115114

116115
/-- The "unlifted" version of multiplication in the colimit. To multiply two dependent pairs
117-
`⟨j₁, x⟩` and `⟨j₂, y⟩`, we pass to a common successor of `j₁` and `j₂` (given by `is_filtered.max`)
116+
`⟨j₁, x⟩` and `⟨j₂, y⟩`, we pass to a common successor of `j₁` and `j₂` (given by `IsFiltered.max`)
118117
and multiply them there.
119118
-/
120119
@[to_additive
121120
"The \"unlifted\" version of addition in the colimit. To add two dependent pairs
122121
`⟨j₁, x⟩` and `⟨j₂, y⟩`, we pass to a common successor of `j₁` and `j₂`
123-
(given by `is_filtered.max`) and add them there."]
122+
(given by `IsFiltered.max`) and add them there."]
124123
noncomputable def colimitMulAux (x y : Σ j, F.obj j) : M.{v, u} F :=
125124
M.mk F ⟨IsFiltered.max x.fst y.fst, F.map (IsFiltered.leftToMax x.1 y.1) x.2 *
126125
F.map (IsFiltered.rightToMax x.1 y.1) y.2
@@ -183,8 +182,8 @@ set_option linter.uppercaseLean3 false in
183182
set_option linter.uppercaseLean3 false in
184183
#align AddMon.filtered_colimits.colimit_add_aux_eq_of_rel_right AddMonCat.FilteredColimits.colimitAddAux_eq_of_rel_right
185184

186-
/-- Multiplication in the colimit. See also `colimit_mul_aux`. -/
187-
@[to_additive "Addition in the colimit. See also `colimit_add_aux`."]
185+
/-- Multiplication in the colimit. See also `colimitMulAux`. -/
186+
@[to_additive "Addition in the colimit. See also `colimitAddAux`."]
188187
noncomputable instance colimitMul : Mul (M.{v, u} F) :=
189188
{ mul := fun x y => by
190189
refine' Quot.lift₂ (colimitMulAux F) _ _ x y
@@ -237,15 +236,15 @@ noncomputable instance colimitMonoid : Monoid (M.{v, u} F) :=
237236
cases' x with j x
238237
rw [colimit_one_eq F j, colimit_mul_mk_eq F ⟨j, 1⟩ ⟨j, x⟩ j (𝟙 j) (𝟙 j), MonoidHom.map_one,
239238
one_mul, F.map_id]
240-
-- Porting note : `id_apply` does not work hear, but the two handsides are def-eq
239+
-- Porting note : `id_apply` does not work here, but the two sides are def-eq
241240
rfl
242241
mul_one := fun x => by
243242
refine Quot.inductionOn x ?_
244243
intro x
245244
cases' x with j x
246245
rw [colimit_one_eq F j, colimit_mul_mk_eq F ⟨j, x⟩ ⟨j, 1⟩ j (𝟙 j) (𝟙 j), MonoidHom.map_one,
247246
mul_one, F.map_id]
248-
-- Porting note : `id_apply` does not work hear, but the two handsides are def-eq
247+
-- Porting note : `id_apply` does not work here, but the two sides are def-eq
249248
rfl
250249
mul_assoc := fun x y z => by
251250
refine Quot.induction_on₃ x y z ?_

Diff for: Mathlib/Algebra/Category/Ring/Limits.lean

+47-46
Original file line numberDiff line numberDiff line change
@@ -49,7 +49,7 @@ instance semiringObj (F : J ⥤ SemiRingCatMax.{v, u}) (j) :
4949
set_option linter.uppercaseLean3 false in
5050
#align SemiRing.semiring_obj SemiRingCat.semiringObj
5151

52-
/-- The flat sections of a functor into `SemiRing` form a subsemiring of all sections.
52+
/-- The flat sections of a functor into `SemiRingCat` form a subsemiring of all sections.
5353
-/
5454
def sectionsSubsemiring (F : J ⥤ SemiRingCatMax.{v, u}) : Subsemiring.{max v u} (∀ j, F.obj j) :=
5555
-- Porting note : if `f` and `g` were inlined, it does not compile
@@ -68,7 +68,7 @@ instance limitSemiring (F : J ⥤ SemiRingCatMax.{v, u}) :
6868
set_option linter.uppercaseLean3 false in
6969
#align SemiRing.limit_semiring SemiRingCat.limitSemiring
7070

71-
/-- `limit.π (F ⋙ forget SemiRing) j` as a `ring_hom`. -/
71+
/-- `limit.π (F ⋙ forget SemiRingCat) j` as a `RingHom`. -/
7272
def limitπRingHom (F : J ⥤ SemiRingCatMax.{v, u}) (j) :
7373
(Types.limitCone.{v, u} (F ⋙ forget SemiRingCat)).pt →+* (F ⋙ forget SemiRingCat).obj j :=
7474
-- Porting note : if `f` and `g` were inlined, it does not compile
@@ -82,10 +82,10 @@ set_option linter.uppercaseLean3 false in
8282

8383
namespace HasLimits
8484

85-
-- The next two definitions are used in the construction of `has_limits SemiRing`.
85+
-- The next two definitions are used in the construction of `HasLimits SemiRingCat`.
8686
-- After that, the limits should be constructed using the generic limits API,
87-
-- e.g. `limit F`, `limit.cone F`, and `limit.is_limit F`.
88-
/-- Construction of a limit cone in `SemiRing`.
87+
-- e.g. `limit F`, `limit.cone F`, and `limit.isLimit F`.
88+
/-- Construction of a limit cone in `SemiRingCat`.
8989
(Internal use only; use the limits API.)
9090
-/
9191
def limitCone (F : J ⥤ SemiRingCatMax.{v, u}) : Cone F where
@@ -97,7 +97,7 @@ def limitCone (F : J ⥤ SemiRingCatMax.{v, u}) : Cone F where
9797
set_option linter.uppercaseLean3 false in
9898
#align SemiRing.has_limits.limit_cone SemiRingCat.HasLimits.limitCone
9999

100-
/-- Witness that the limit cone in `SemiRing` is a limit cone.
100+
/-- Witness that the limit cone in `SemiRingCat` is a limit cone.
101101
(Internal use only; use the limits API.)
102102
-/
103103
def limitConeIsLimit (F : J ⥤ SemiRingCatMax.{v, u}) : IsLimit (limitCone F) := by
@@ -139,8 +139,8 @@ set_option linter.uppercaseLean3 false in
139139
/-- The forgetful functor from semirings to additive commutative monoids preserves all limits.
140140
-/
141141
instance forget₂AddCommMonPreservesLimitsOfSize :
142-
PreservesLimitsOfSize.{v, v} (forget₂ SemiRingCat AddCommMonCat.{max v u})
143-
where preservesLimitsOfShape {_ _} :=
142+
PreservesLimitsOfSize.{v, v} (forget₂ SemiRingCat AddCommMonCat.{max v u}) where
143+
preservesLimitsOfShape {_ _} :=
144144
{ preservesLimit := fun {F} =>
145145
preservesLimitOfPreservesLimitCone (limitConeIsLimit.{v, u} F)
146146
(forget₂AddCommMonPreservesLimitsAux F) }
@@ -164,8 +164,8 @@ set_option linter.uppercaseLean3 false in
164164
/-- The forgetful functor from semirings to monoids preserves all limits.
165165
-/
166166
instance forget₂MonPreservesLimitsOfSize :
167-
PreservesLimitsOfSize.{v, v} (forget₂ SemiRingCat MonCat.{max v u})
168-
where preservesLimitsOfShape {_ _} :=
167+
PreservesLimitsOfSize.{v, v} (forget₂ SemiRingCat MonCat.{max v u}) where
168+
preservesLimitsOfShape {_ _} :=
169169
{ preservesLimit := fun {F} =>
170170
preservesLimitOfPreservesLimitCone (limitConeIsLimit F)
171171
(forget₂MonPreservesLimitsAux.{v, u} F) }
@@ -179,8 +179,9 @@ set_option linter.uppercaseLean3 false in
179179

180180
/-- The forgetful functor from semirings to types preserves all limits.
181181
-/
182-
instance forgetPreservesLimitsOfSize : PreservesLimitsOfSize.{v, v} (forget SemiRingCat.{max v u})
183-
where preservesLimitsOfShape {_ _} :=
182+
instance forgetPreservesLimitsOfSize :
183+
PreservesLimitsOfSize.{v, v} (forget SemiRingCat.{max v u}) where
184+
preservesLimitsOfShape {_ _} :=
184185
{ preservesLimit := fun {F} =>
185186
preservesLimitOfPreservesLimitCone (limitConeIsLimit F)
186187
(Types.limitConeIsLimit.{v, u} (F ⋙ forget _)) }
@@ -217,15 +218,15 @@ instance limitCommSemiring (F : J ⥤ CommSemiRingCatMax.{v, u}) :
217218
set_option linter.uppercaseLean3 false in
218219
#align CommSemiRing.limit_comm_semiring CommSemiRingCat.limitCommSemiring
219220

220-
/-- We show that the forgetful functor `CommSemiRingSemiRing` creates limits.
221+
/-- We show that the forgetful functor `CommSemiRingCatSemiRingCat` creates limits.
221222
222-
All we need to do is notice that the limit point has a `comm_semiring` instance available,
223+
All we need to do is notice that the limit point has a `CommSemiring` instance available,
223224
and then reuse the existing limit.
224225
-/
225226
instance (F : J ⥤ CommSemiRingCatMax.{v, u}) :
226227
CreatesLimit F (forget₂ CommSemiRingCatMax.{v, u} SemiRingCatMax.{v, u}) :=
227-
-- Porting note : `CommSemiRing ⥤ Type` reflecting isomorphism is needed to make Lean see that
228-
-- `CommSemiRingCat ⥤ SemiRingCat` reflects isomorphism. `CommSemiRing ⥤ Type` reflecting
228+
-- Porting note : `CommSemiRingCat ⥤ Type` reflecting isomorphism is needed to make Lean see that
229+
-- `CommSemiRingCat ⥤ SemiRingCat` reflects isomorphism. `CommSemiRingCat ⥤ Type` reflecting
229230
-- isomorphism is added manually since Lean can't see it, but even with this addition Lean can not
230231
-- see `CommSemiRingCat ⥤ SemiRingCat` reflects isomorphism, so this instance is also added.
231232
letI : ReflectsIsomorphisms (forget CommSemiRingCatMax.{v, u}) :=
@@ -253,7 +254,7 @@ instance (F : J ⥤ CommSemiRingCatMax.{v, u}) :
253254
fun x y => Subtype.ext <| funext fun j => by exact (s.π.app j).map_add x y⟩)
254255
fun s => rfl }
255256

256-
/-- A choice of limit cone for a functor into `CommSemiRing`.
257+
/-- A choice of limit cone for a functor into `CommSemiRingCat`.
257258
(Generally, you'll just want to use `limit F`.)
258259
-/
259260
def limitCone (F : J ⥤ CommSemiRingCatMax.{v, u}) : Cone F :=
@@ -272,8 +273,7 @@ set_option linter.uppercaseLean3 false in
272273
/- ./././Mathport/Syntax/Translate/Command.lean:322:38: unsupported irreducible non-definition -/
273274
/-- The category of rings has all limits. -/
274275
instance hasLimitsOfSize : HasLimitsOfSize.{v, v} CommSemiRingCatMax.{v, u} :=
275-
{
276-
has_limits_of_shape := fun _ _ =>
276+
{ has_limits_of_shape := fun _ _ =>
277277
{ has_limit := fun F =>
278278
hasLimit_of_created F (forget₂ CommSemiRingCat SemiRingCatMax.{v, u}) } }
279279
set_option linter.uppercaseLean3 false in
@@ -287,8 +287,8 @@ set_option linter.uppercaseLean3 false in
287287
/-- The forgetful functor from rings to semirings preserves all limits.
288288
-/
289289
instance forget₂SemiRingPreservesLimitsOfSize :
290-
PreservesLimitsOfSize.{v, v} (forget₂ CommSemiRingCat SemiRingCat.{max v u})
291-
where preservesLimitsOfShape {_ _} :=
290+
PreservesLimitsOfSize.{v, v} (forget₂ CommSemiRingCat SemiRingCat.{max v u}) where
291+
preservesLimitsOfShape {_ _} :=
292292
{ preservesLimit := fun {F} =>
293293
preservesLimitOfPreservesLimitCone (limitConeIsLimit.{v, u} F)
294294
(SemiRingCat.HasLimits.limitConeIsLimit _) }
@@ -305,8 +305,8 @@ set_option linter.uppercaseLean3 false in
305305
types could have been computed instead as limits in the category of types.)
306306
-/
307307
instance forgetPreservesLimitsOfSize :
308-
PreservesLimitsOfSize.{v, v} (forget CommSemiRingCatMax.{v, u})
309-
where preservesLimitsOfShape {_ _} :=
308+
PreservesLimitsOfSize.{v, v} (forget CommSemiRingCatMax.{v, u}) where
309+
preservesLimitsOfShape {_ _} :=
310310
{ preservesLimit := fun {F} =>
311311
preservesLimitOfPreservesLimitCone (limitConeIsLimit.{v, u} F)
312312
(Types.limitConeIsLimit.{v, u} _) }
@@ -321,7 +321,7 @@ set_option linter.uppercaseLean3 false in
321321
end CommSemiRingCat
322322

323323
-- Porting note: typemax hack to fix universe complaints
324-
/-- An alias for `Ring.{max u v}`, to deal around unification issues. -/
324+
/-- An alias for `RingCat.{max u v}`, to deal around unification issues. -/
325325
@[nolint checkUnivs]
326326
abbrev RingCatMax.{u1, u2} := RingCat.{max u1 u2}
327327

@@ -335,7 +335,7 @@ instance ringObj (F : J ⥤ RingCatMax.{v, u}) (j) : Ring ((F ⋙ forget RingCat
335335
set_option linter.uppercaseLean3 false in
336336
#align Ring.ring_obj RingCat.ringObj
337337

338-
/-- The flat sections of a functor into `Ring` form a subring of all sections.
338+
/-- The flat sections of a functor into `RingCat` form a subring of all sections.
339339
-/
340340
def sectionsSubring (F : J ⥤ RingCatMax.{v, u}) : Subring.{max v u} (∀ j, F.obj j) :=
341341
letI f : J ⥤ AddGroupCat.{max v u} :=
@@ -354,13 +354,13 @@ instance limitRing (F : J ⥤ RingCatMax.{v, u}) :
354354
set_option linter.uppercaseLean3 false in
355355
#align Ring.limit_ring RingCat.limitRing
356356

357-
/-- We show that the forgetful functor `CommRingRing` creates limits.
357+
/-- We show that the forgetful functor `CommRingCatRingCat` creates limits.
358358
359-
All we need to do is notice that the limit point has a `ring` instance available,
359+
All we need to do is notice that the limit point has a `Ring` instance available,
360360
and then reuse the existing limit.
361361
-/
362362
instance (F : J ⥤ RingCatMax.{v, u}) :
363-
CreatesLimit F (forget₂ RingCatMax.{v, u} SemiRingCatMax.{v, u}) :=
363+
CreatesLimit F (forget₂ RingCatMax.{v, u} SemiRingCatMax.{v, u}) :=
364364
letI : ReflectsIsomorphisms (forget₂ RingCatMax SemiRingCatMax) :=
365365
CategoryTheory.reflectsIsomorphisms_forget₂ _ _
366366
letI c : Cone F :=
@@ -376,7 +376,7 @@ instance (F : J ⥤ RingCatMax.{v, u}) :
376376
IsLimit.ofFaithful (forget₂ RingCat SemiRingCat.{max v u})
377377
(by apply SemiRingCat.HasLimits.limitConeIsLimit _) (fun s => _) fun s => rfl }
378378

379-
/-- A choice of limit cone for a functor into `Ring`.
379+
/-- A choice of limit cone for a functor into `RingCat`.
380380
(Generally, you'll just want to use `limit F`.)
381381
-/
382382
def limitCone (F : J ⥤ RingCatMax.{v, u}) : Cone F :=
@@ -409,8 +409,8 @@ set_option linter.uppercaseLean3 false in
409409
/-- The forgetful functor from rings to semirings preserves all limits.
410410
-/
411411
instance forget₂SemiRingPreservesLimitsOfSize :
412-
PreservesLimitsOfSize.{v, v} (forget₂ RingCat SemiRingCat.{max v u})
413-
where preservesLimitsOfShape {_ _} :=
412+
PreservesLimitsOfSize.{v, v} (forget₂ RingCat SemiRingCat.{max v u}) where
413+
preservesLimitsOfShape {_ _} :=
414414
{ preservesLimit := fun {F} =>
415415
preservesLimitOfPreservesLimitCone (limitConeIsLimit.{v, u} F)
416416
(SemiRingCat.HasLimits.limitConeIsLimit.{v, u} _) }
@@ -435,8 +435,8 @@ set_option linter.uppercaseLean3 false in
435435
/-- The forgetful functor from rings to additive commutative groups preserves all limits.
436436
-/
437437
instance forget₂AddCommGroupPreservesLimitsOfSize :
438-
PreservesLimitsOfSize.{v, v} (forget₂ RingCatMax.{v, u} AddCommGroupCat.{max v u})
439-
where preservesLimitsOfShape {_ _} :=
438+
PreservesLimitsOfSize.{v, v} (forget₂ RingCatMax.{v, u} AddCommGroupCat.{max v u}) where
439+
preservesLimitsOfShape {_ _} :=
440440
{ preservesLimit := fun {F} =>
441441
preservesLimitOfPreservesLimitCone (limitConeIsLimit.{v, u} F)
442442
(forget₂AddCommGroupPreservesLimitsAux F) }
@@ -452,8 +452,8 @@ set_option linter.uppercaseLean3 false in
452452
/-- The forgetful functor from rings to types preserves all limits. (That is, the underlying
453453
types could have been computed instead as limits in the category of types.)
454454
-/
455-
instance forgetPreservesLimitsOfSize : PreservesLimitsOfSize.{v, v} (forget RingCatMax.{v, u})
456-
where preservesLimitsOfShape {_ _} :=
455+
instance forgetPreservesLimitsOfSize : PreservesLimitsOfSize.{v, v} (forget RingCatMax.{v, u}) where
456+
preservesLimitsOfShape {_ _} :=
457457
{ preservesLimit := fun {F} =>
458458
preservesLimitOfPreservesLimitCone (limitConeIsLimit.{v, u} F)
459459
(Types.limitConeIsLimit.{v, u} _) }
@@ -468,7 +468,7 @@ set_option linter.uppercaseLean3 false in
468468
end RingCat
469469

470470
-- Porting note: typemax hack to fix universe complaints
471-
/-- An alias for `CommRing.{max u v}`, to deal around unification issues. -/
471+
/-- An alias for `CommRingCat.{max u v}`, to deal around unification issues. -/
472472
@[nolint checkUnivs]
473473
abbrev CommRingCatMax.{u1, u2} := CommRingCat.{max u1 u2}
474474

@@ -490,17 +490,17 @@ instance limitCommRing (F : J ⥤ CommRingCatMax.{v, u}) :
490490
set_option linter.uppercaseLean3 false in
491491
#align CommRing.limit_comm_ring CommRingCat.limitCommRing
492492

493-
/-- We show that the forgetful functor `CommRingRing` creates limits.
493+
/-- We show that the forgetful functor `CommRingCatRingCat` creates limits.
494494
495-
All we need to do is notice that the limit point has a `comm_ring` instance available,
495+
All we need to do is notice that the limit point has a `CommRing` instance available,
496496
and then reuse the existing limit.
497497
-/
498498
instance (F : J ⥤ CommRingCatMax.{v, u}) :
499499
CreatesLimit F (forget₂ CommRingCatMax.{v, u} RingCatMax.{v, u}) :=
500500
/-
501501
A terse solution here would be
502502
```
503-
creates_limit_of_fully_faithful_of_iso (CommRing.of (limit (F ⋙ forget _))) (iso.refl _)
503+
createsLimitOfFullyFaithfulOfIso (CommRingCat.of (limit (F ⋙ forget _))) (Iso.refl _)
504504
```
505505
but it seems this would introduce additional identity morphisms in `limit.π`.
506506
-/
@@ -531,7 +531,7 @@ instance (F : J ⥤ CommRingCatMax.{v, u}) :
531531
(F ⋙ forget₂ CommRingCatMax.{v, u} RingCatMax.{v, u})).lift
532532
((forget₂ _ RingCatMax.{v, u}).mapCone s)) fun _ => rfl }
533533

534-
/-- A choice of limit cone for a functor into `CommRing`.
534+
/-- A choice of limit cone for a functor into `CommRingCat`.
535535
(Generally, you'll just want to use `limit F`.)
536536
-/
537537
def limitCone (F : J ⥤ CommRingCatMax.{v, u}) : Cone F :=
@@ -569,8 +569,8 @@ set_option linter.uppercaseLean3 false in
569569
(That is, the underlying rings could have been computed instead as limits in the category of rings.)
570570
-/
571571
instance forget₂RingPreservesLimitsOfSize :
572-
PreservesLimitsOfSize.{v, v} (forget₂ CommRingCat RingCat.{max v u})
573-
where preservesLimitsOfShape {_ _} :=
572+
PreservesLimitsOfSize.{v, v} (forget₂ CommRingCat RingCat.{max v u}) where
573+
preservesLimitsOfShape {_ _} :=
574574
{ preservesLimit := fun {F} =>
575575
preservesLimitOfPreservesLimitCone.{v, v} (limitConeIsLimit.{v, u} F)
576576
(RingCat.limitConeIsLimit.{v, u} _) }
@@ -595,8 +595,8 @@ set_option linter.uppercaseLean3 false in
595595
in the category of commutative semirings.)
596596
-/
597597
instance forget₂CommSemiRingPreservesLimitsOfSize :
598-
PreservesLimitsOfSize.{v, v} (forget₂ CommRingCat CommSemiRingCat.{max v u})
599-
where preservesLimitsOfShape {_ _} :=
598+
PreservesLimitsOfSize.{v, v} (forget₂ CommRingCat CommSemiRingCat.{max v u}) where
599+
preservesLimitsOfShape {_ _} :=
600600
{ preservesLimit := fun {F} =>
601601
preservesLimitOfPreservesLimitCone (limitConeIsLimit.{v, u} F)
602602
(forget₂CommSemiRingPreservesLimitsAux.{v, u} F) }
@@ -612,8 +612,9 @@ set_option linter.uppercaseLean3 false in
612612
/-- The forgetful functor from commutative rings to types preserves all limits.
613613
(That is, the underlying types could have been computed instead as limits in the category of types.)
614614
-/
615-
instance forgetPreservesLimitsOfSize : PreservesLimitsOfSize.{v, v} (forget CommRingCat.{max v u})
616-
where preservesLimitsOfShape {_ _} :=
615+
instance forgetPreservesLimitsOfSize :
616+
PreservesLimitsOfSize.{v, v} (forget CommRingCat.{max v u}) where
617+
preservesLimitsOfShape {_ _} :=
617618
{ preservesLimit := fun {F} =>
618619
preservesLimitOfPreservesLimitCone.{v, v} (limitConeIsLimit.{v, u} F)
619620
(Types.limitConeIsLimit.{v, u} _) }

Diff for: Mathlib/Algebra/Free.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -483,7 +483,7 @@ theorem mk_mul_mk (x y : α) (L1 L2 : List α) : mk x L1 * mk y L2 = mk x (L1 ++
483483
#align free_semigroup.mk_mul_mk FreeSemigroup.mk_mul_mk
484484

485485
/-- The embedding `α → FreeSemigroup α`. -/
486-
@[to_additive (attr := simps) "The embedding `α → free_add_semigroup α`."]
486+
@[to_additive (attr := simps) "The embedding `α → FreeAddSemigroup α`."]
487487
def of (x : α) : FreeSemigroup α := ⟨x, []⟩
488488
#align free_semigroup.of FreeSemigroup.of
489489

0 commit comments

Comments
 (0)