We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 409aebc commit 2cf26daCopy full SHA for 2cf26da
Mathlib/CategoryTheory/Monoidal/Cartesian/Mon_.lean
@@ -355,3 +355,13 @@ lemma MonObj.mul_eq_mul : μ = fst M M * snd _ _ :=
355
show _ = _ ≫ _ by rw [lift_fst_snd, Category.id_comp]
356
357
@[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