Skip to content

Commit 6398d18

Browse files
committed
feat: tensor product of group objects (#29134)
... and similarly for commutative monoid objects. From Toric
1 parent 4aa8d32 commit 6398d18

File tree

2 files changed

+21
-3
lines changed

2 files changed

+21
-3
lines changed

Mathlib/CategoryTheory/Monoidal/Grp_.lean

Lines changed: 9 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -252,11 +252,17 @@ lemma toMon_Class_injective {X : C} :
252252
exacts [congr(($e.symm).mul), congr(($e.symm).one)]
253253

254254
@[ext]
255-
lemma _root_.Grp_Class.ext {X : C} (h₁ h₂ : Grp_Class X)
256-
(H : h₁.toMon_Class = h₂.toMon_Class) : h₁ = h₂ :=
255+
lemma ext {X : C} (h₁ h₂ : Grp_Class X) (H : h₁.toMon_Class = h₂.toMon_Class) : h₁ = h₂ :=
257256
Grp_Class.toMon_Class_injective H
258257

259-
end Grp_Class
258+
namespace tensorObj
259+
variable [BraidedCategory C] {G H : C} [Grp_Class G] [Grp_Class H]
260+
261+
@[simps inv]
262+
instance : Grp_Class (G ⊗ H) where
263+
inv := ι ⊗ₘ ι
264+
265+
end Grp_Class.tensorObj
260266

261267
namespace Grp_
262268

Mathlib/CategoryTheory/Monoidal/Mon_.lean

Lines changed: 12 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -942,6 +942,18 @@ lemma Mon_Class.mul_mul_mul_comm' [IsCommMon M] :
942942

943943
end
944944

945+
section SymmetricCategory
946+
variable [SymmetricCategory C] {M N W X Y Z : C} [Mon_Class M] [Mon_Class N]
947+
948+
instance [IsCommMon M] [IsCommMon N] : IsCommMon (M ⊗ N) where
949+
mul_comm := by
950+
simp [← IsIso.inv_comp_eq, tensorμ, ← associator_inv_naturality_left_assoc,
951+
← associator_naturality_right_assoc, SymmetricCategory.braiding_swap_eq_inv_braiding M N,
952+
← tensorHom_def_assoc, -whiskerRight_tensor, -tensor_whiskerLeft, ← tensor_comp,
953+
Mon_Class.tensorObj.mul_def, ← whiskerLeft_comp_assoc, -whiskerLeft_comp]
954+
955+
end SymmetricCategory
956+
945957
/-!
946958
Projects:
947959
* Check that `Mon_ MonCat ≌ CommMonCat`, via the Eckmann-Hilton argument.

0 commit comments

Comments
 (0)