Skip to content

Commit

Permalink
refactor: Generalize RingHom.coe_mk & RingHom.coe_monoidHom_mk (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
Komyyy committed Feb 20, 2023
1 parent 200a85b commit 5c2c900
Showing 1 changed file with 2 additions and 3 deletions.
5 changes: 2 additions & 3 deletions Mathlib/Algebra/Hom/Ring.lean
Expand Up @@ -464,7 +464,7 @@ theorem toFun_eq_coe (f : α →+* β) : f.toFun = f :=
#align ring_hom.to_fun_eq_coe RingHom.toFun_eq_coe

@[simp]
theorem coe_mk (f : α → β) (h₁ h₂ h₃ h₄) : ⇑(⟨⟨⟨f, h₁, h₂⟩, h₃, h₄⟩ : α →+* β) = f :=
theorem coe_mk (f : α →* β) (h₁ h₂) : ((⟨f, h₁, h₂⟩ : α →+* β) : α → β) = f :=
rfl
#align ring_hom.coe_mk RingHom.coe_mk

Expand Down Expand Up @@ -494,8 +494,7 @@ theorem toMonoidWithZeroHom_eq_coe (f : α →+* β) : (f.toMonoidWithZeroHom :
#align ring_hom.to_monoid_with_zero_hom_eq_coe RingHom.toMonoidWithZeroHom_eq_coe

@[simp]
theorem coe_monoidHom_mk (f : α → β) (h₁ h₂ h₃ h₄) :
((⟨⟨⟨f, h₁⟩, h₂⟩, h₃, h₄⟩ : α →+* β) : α →* β) = ⟨⟨f, h₁⟩, h₂⟩ :=
theorem coe_monoidHom_mk (f : α →* β) (h₁ h₂) : ((⟨f, h₁, h₂⟩ : α →+* β) : α →* β) = f :=
rfl
#align ring_hom.coe_monoid_hom_mk RingHom.coe_monoidHom_mk

Expand Down

0 comments on commit 5c2c900

Please sign in to comment.