Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 02cdc33

Browse files
committed
chore(algebra/group/hom): Add missing simp lemmas (#4958)
These are named in the same pattern as `linear_map.to_add_monoid_hom_coe`
1 parent 3d6291e commit 02cdc33

File tree

1 file changed

+7
-0
lines changed

1 file changed

+7
-0
lines changed

src/algebra/group/hom.lean

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -130,6 +130,13 @@ lemma mul_hom.coe_mk [has_mul M] [has_mul N]
130130
lemma monoid_hom.coe_mk [monoid M] [monoid N]
131131
(f : M → N) (h1 hmul) : ⇑(monoid_hom.mk f h1 hmul) = f := rfl
132132

133+
@[simp, to_additive]
134+
lemma monoid_hom.to_one_hom_coe [monoid M] [monoid N] (f : M →* N) :
135+
(f.to_one_hom : M → N) = f := rfl
136+
@[simp, to_additive]
137+
lemma monoid_hom.to_mul_hom_coe [monoid M] [monoid N] (f : M →* N) :
138+
(f.to_mul_hom : M → N) = f := rfl
139+
133140
@[to_additive]
134141
theorem one_hom.congr_fun [has_one M] [has_one N]
135142
{f g : one_hom M N} (h : f = g) (x : M) : f x = g x :=

0 commit comments

Comments
 (0)