mathlib
mathlib copied to clipboard
Make `to_ring_hom_eq_coe` into a `simp` lemma in `ring_equiv`
Right now to_ring_hom_eq_coe is not a simp lemma, which makes it not possible to deduce something like (f : R ≃+* S) : ⇑(f.to_ring_hom) = ⇑f by simp. The open question is whether f.to_ring_hom or ↑f should be simp-normal-form.
This came up in this thread in zulip