Skip to content

Commit 2cf26da

Browse files
committed
feat: isomorphic monoid objects have isomorphic hom monoids (#29830)
From Toric
1 parent 409aebc commit 2cf26da

File tree

1 file changed

+10
-0
lines changed
  • Mathlib/CategoryTheory/Monoidal/Cartesian

1 file changed

+10
-0
lines changed

Mathlib/CategoryTheory/Monoidal/Cartesian/Mon_.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -355,3 +355,13 @@ lemma MonObj.mul_eq_mul : μ = fst M M * snd _ _ :=
355355
show _ = _ ≫ _ by rw [lift_fst_snd, Category.id_comp]
356356

357357
@[deprecated (since := "2025-09-09")] alias Mon_Class.mul_eq_mul := MonObj.mul_eq_mul
358+
359+
namespace Hom
360+
361+
/-- If `M` and `N` are isomorphic as monoid objects, then `X ⟶ M` and `X ⟶ N` are isomorphic
362+
monoids. -/
363+
@[simps!]
364+
def mulEquivCongrRight (e : M ≅ N) [IsMonHom e.hom] (X : C) : (X ⟶ M) ≃* (X ⟶ N) :=
365+
((yonedaMon.mapIso <| Mon.mkIso' e).app <| .op X).monCatIsoToMulEquiv
366+
367+
end Hom

0 commit comments

Comments
 (0)