Zulip Chat Archive
Stream: general
Topic: option lemma
Patrick Massot (Dec 29 2021 at 21:14):
Is it possible that
@[simp] lemma option.mem_some_iff {α : Type*} {a b : α} : a ∈ some b ↔ b = a :=
by { rw [option.mem_iff], exact option.some_inj }
is missing? @Mario Carneiro ?
Patrick Massot (Dec 29 2021 at 21:15):
Is there a reason not to do that?
Yaël Dillies (Dec 29 2021 at 21:17):
I have this lemma on a branch! Definitely useful.
Patrick Massot (Dec 29 2021 at 21:17):
There is something weird going on. If I try to put this in its natural place then simp
does it already
Adam Topaz (Dec 29 2021 at 21:23):
Patrick Massot (Dec 29 2021 at 21:23):
This is not exactly the same
Adam Topaz (Dec 29 2021 at 21:23):
I know, but that's the lemma that is used by simp, at least on my machine.
Patrick Massot (Dec 29 2021 at 21:25):
I added the missing lemma without the simp
attribute, so it can't hurt.
Last updated: Dec 20 2023 at 11:08 UTC