Zulip Chat Archive
Stream: Is there code for X?
Topic: set singletons injective
Joachim Breitner (Jan 13 2022 at 15:57):
I can’t find a lemma for function.injective (λ (x : B), {x})
. Insufficient search ability, or does that not exist for some reasons (e.g. because this is a very classical view on sets)?
(I found a different way to do my proof, so not super important.)
Yaël Dillies (Jan 13 2022 at 16:10):
docs#finset.singleton_injective
Yaël Dillies (Jan 13 2022 at 16:10):
and it seems we're missing the set
version?
Joachim Breitner (Jan 13 2022 at 16:10):
Somehow that didn't work for me; it’s for finset
and I needed set
.
Eric Wieser (Jan 13 2022 at 16:32):
Yeah, I agree that docs#set.singleton_injective is missing. Want to PR it, @Joachim Breitner? The proof ought to be trivial
Eric Wieser (Jan 13 2022 at 16:33):
(note the statement is better as lemma singleton_injective : injective (singleton : α → set α)
as this doesn't introduce unnecessary λ
binders)
Eric Wieser (Jan 13 2022 at 16:34):
It belongs right before docs#set.singleton_eq_singleton_iff
Joachim Breitner (Jan 14 2022 at 15:43):
I’ll give it a shot later
Last updated: Dec 20 2023 at 11:08 UTC