Zulip Chat Archive

Stream: Is there code for X?

Topic: bijective function between types of equal cardinality


Eric Wieser (Apr 30 2022 at 23:22):

Did you forget to include the signature you're asking about? (edit: I renamed the thread now that you've posted your actual question)

Joseph O (May 01 2022 at 00:07):

Oh yeah i forgot.

theorem card_a_eq_card_b_iff_bijective {α β : Type} (f : α  β) : #α = #β  function.bijective f :=
begin
  sorry,
end

Joseph O (May 01 2022 at 00:08):

I really just want a better name for this.

Kyle Miller (May 01 2022 at 00:12):

That theorem's not true -- f doesn't have to be bijective if the cardinalities of the domain and codomain are the same.

Eric Wieser (May 01 2022 at 00:13):

Example: set α = β = ℕ and f = 0

Eric Wieser (May 01 2022 at 00:14):

I would guess the statement you want is docs#cardinal.eq, which is essentially true by definition

Eric Wieser (May 01 2022 at 00:15):

Turn an equiv into a bijective function is easy and not really a useful thing to do anyway


Last updated: Dec 20 2023 at 11:08 UTC