Zulip Chat Archive
Stream: Is there code for X?
Topic: missing simp lemma for `EquivLike`
Jireh Loreaux (Jan 16 2024 at 04:28):
Do we agree that (a) this is missing, and (b) we want it?
import Mathlib.Logic.Equiv.Defs
@[simp, norm_cast]
theorem EquivLike.coe_symm_toEquiv {α β F : Sort*} [EquivLike F α β] (e : F) :
⇑(e : α ≃ β).symm = EquivLike.inv e := rfl
Jireh Loreaux (Jan 16 2024 at 13:47):
Nevermind.
Richard Copley (Jan 16 2024 at 14:13):
symm_apply? Never mind.
Floris van Doorn (Jan 16 2024 at 14:30):
I think that we usually prefer ⇑(e : α ≃ β).symm
as the simp-normal form, not EquivLike.inv e
.
Floris van Doorn (Jan 16 2024 at 14:32):
E.g. docs#Equiv.invFun_as_coe is a simp-lemma.
Jireh Loreaux (Jan 16 2024 at 15:46):
Yeah, sorry. For some reason something was broken, I added this and it was fixed. But then it turned out that I misdiagnosed.
Last updated: May 02 2025 at 03:31 UTC