Commit 2025-06-04 18:15 ac1246f8

View on Github →

feat(CategoryTheory/Monoidal): define Mon_ by using Mon_Class (#24646) The main change is from

structure Mon_ where
  X : C
  one : 𝟙_ C ⟶ X
  mul : X ⊗ X ⟶ X
  one_mul : (one ▷ X) ≫ mul = (λ_ X).hom := by aesop_cat
  mul_one : (X ◁ one) ≫ mul = (ρ_ X).hom := by aesop_cat
  mul_assoc : (mul ▷ X) ≫ mul = (α_ X X X).hom ≫ (X ◁ mul) ≫ mul := by aesop_cat

to

structure Mon_ where
  X : C
  [mon : Mon_Class X]

Estimated changes

deleted theorem Grp_.eq_lift_inv_left
deleted theorem Grp_.eq_lift_inv_right
modified theorem Grp_.forget₂Mon_obj_mul
modified theorem Grp_.forget₂Mon_obj_one
deleted theorem Grp_.inv_comp_inv
deleted theorem Grp_.inv_hom
deleted theorem Grp_.inv_inv
deleted theorem Grp_.isPullback
deleted theorem Grp_.lift_comp_inv_left
deleted theorem Grp_.lift_comp_inv_right
deleted theorem Grp_.lift_inv_comp_left
deleted theorem Grp_.lift_inv_comp_right
deleted theorem Grp_.lift_inv_left_eq
deleted theorem Grp_.lift_inv_right_eq
deleted theorem Grp_.lift_left_mul_ext
deleted def Grp_.mulRight
deleted theorem Grp_.mulRight_one
deleted theorem Grp_.mul_inv
added def Grp_.toMon_
modified structure Grp_
added theorem Grp_Class.inv_comp_inv
added theorem Grp_Class.inv_hom
added theorem Grp_Class.inv_inv
added theorem Grp_Class.isPullback
added theorem Grp_Class.mulRight_one
added theorem Grp_Class.mul_inv
deleted theorem IsMon_Hom.inv_hom