File tree Expand file tree Collapse file tree 2 files changed +34
-0
lines changed
Mathlib/CategoryTheory/Monoidal Expand file tree Collapse file tree 2 files changed +34
-0
lines changed Original file line number Diff line number Diff line change @@ -233,3 +233,18 @@ def equivLaxBraidedFunctorPUnit : LaxBraidedFunctor (Discrete PUnit.{u + 1}) C
233
233
counitIso := counitIso C
234
234
235
235
end CommMon_
236
+
237
+ namespace CommMon_
238
+
239
+ variable {C}
240
+
241
+ /-- Construct an object of `CommMon_ C` from an object `X : C` a `Mon_Class X` instance
242
+ and a `IsCommMon X` insance. -/
243
+ def mk' (X : C) [Mon_Class X] [IsCommMon X] : CommMon_ C where
244
+ __ := Mon_.mk' X
245
+ mul_comm := IsCommMon.mul_comm X
246
+
247
+ instance (X : CommMon_ C) : IsCommMon X.X where
248
+ mul_comm' := X.mul_comm
249
+
250
+ end CommMon_
Original file line number Diff line number Diff line change @@ -671,6 +671,25 @@ end SymmetricCategory
671
671
672
672
end Mon_
673
673
674
+ section
675
+
676
+ variable {C} [BraidedCategory.{v₁} C]
677
+
678
+ /-- Predicate for a monoid object to be commutative. -/
679
+ class IsCommMon (X : C) [Mon_Class X] where
680
+ mul_comm' : (β_ X X).hom ≫ μ = μ := by aesop_cat
681
+
682
+ open scoped Mon_Class
683
+
684
+ namespace IsCommMon
685
+
686
+ @[reassoc (attr := simp)]
687
+ theorem mul_comm (X : C) [Mon_Class X] [IsCommMon X] : (β_ X X).hom ≫ μ = μ := mul_comm'
688
+
689
+ end IsCommMon
690
+
691
+ end
692
+
674
693
/-!
675
694
Projects:
676
695
* Check that `Mon_ MonCat ≌ CommMonCat`, via the Eckmann-Hilton argument.
You can’t perform that action at this time.
0 commit comments