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

Commit d2cc044

Browse files
committed
chore(algebra/algebra/basic): add a missing coe lemma (#6535)
This is just to stop the terrible pain of having to work with `⇑(e.to_ring_equiv) x` in goals. In the long run, we should sort out the simp normal form, but for now I just want to stop the pain.
1 parent ef1a00b commit d2cc044

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

src/algebra/algebra/basic.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -673,7 +673,9 @@ rfl
673673

674674
@[simp] lemma to_fun_eq_coe (e : A₁ ≃ₐ[R] A₂) : e.to_fun = e := rfl
675675

676+
-- TODO: decide on a simp-normal form so that only one of these two lemmas is needed
676677
@[simp, norm_cast] lemma coe_ring_equiv : ((e : A₁ ≃+* A₂) : A₁ → A₂) = e := rfl
678+
@[simp] lemma coe_ring_equiv' : (e.to_ring_equiv : A₁ → A₂) = e := rfl
677679

678680
lemma coe_ring_equiv_injective : function.injective (λ e : A₁ ≃ₐ[R] A₂, (e : A₁ ≃+* A₂)) :=
679681
begin

0 commit comments

Comments
 (0)