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

Commit fb815d7

Browse files
committed
feat(algebra/ring/basic): coercions of ring_hom.id (#8439)
Two basic lemmas about the identity map as a ring hom, split off from #3292 at @eric-wieser's suggestion.
1 parent e9309e3 commit fb815d7

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

src/algebra/ring/basic.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -462,6 +462,8 @@ include rα
462462
instance : inhabited (α →+* α) := ⟨id α⟩
463463

464464
@[simp] lemma id_apply (x : α) : ring_hom.id α x = x := rfl
465+
@[simp] lemma coe_add_monoid_hom_id : (id α : α →+ α) = add_monoid_hom.id α := rfl
466+
@[simp] lemma coe_monoid_hom_id : (id α : α →* α) = monoid_hom.id α := rfl
465467

466468
variable {rγ : non_assoc_semiring γ}
467469
include rβ rγ

0 commit comments

Comments
 (0)