Zulip Chat Archive
Stream: Is there code for X?
Topic: no injective function on `ordinal`
Sebastien Gouezel (Sep 28 2021 at 13:22):
Is there already a lemma saying that ordinal.{u}
is bigger than any type in Type u
?
lemma foo {β : Type u} (f : ordinal.{u} → β) : ¬ (function.injective f) :=
Reid Barton (Sep 28 2021 at 13:26):
Last updated: Dec 20 2023 at 11:08 UTC