Zulip Chat Archive
Stream: Is there code for X?
Topic: mem_iff for subsingletons
Yaël Dillies (Sep 03 2021 at 13:55):
Do we already have this simple lemma somewhere?
@[simp] lemma set.mem_iff_nonempty_of_subsingleton {α : Type*} [subsingleton α] {s : set α}
{x : α} :
x ∈ s ↔ s.nonempty :=
begin
refine ⟨λ hx, ⟨x, hx⟩, _⟩,
rintro ⟨y, hy⟩,
rwa subsingleton.elim x y,
end
Scott Morrison (Sep 03 2021 at 23:26):
It's not super clear this should be a simp lemma.
Last updated: Dec 20 2023 at 11:08 UTC