Skip to content

Commit

Permalink
feat(data/complex/basic): #ℂ = 𝔠 (#12871)
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Mar 24, 2022
1 parent 584ae9d commit 7967128
Showing 1 changed file with 30 additions and 0 deletions.
30 changes: 30 additions & 0 deletions src/data/complex/cardinality.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,30 @@
/-
Copyright (c) 2022 Violeta Hernández Palacios. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Violeta Hernández Palacios
-/

import data.complex.basic
import data.real.cardinality

/-!
# The cardinality of the complex numbers
This file shows that the complex numbers have cardinality continuum, i.e. `#ℂ = 𝔠`.
-/

open cardinal set

open_locale cardinal

/-- The cardinality of the complex numbers, as a type. -/
@[simp] theorem mk_complex : #ℂ = 𝔠 :=
by rw [mk_congr complex.equiv_real_prod, mk_prod, lift_id, mk_real, continuum_mul_self]

/-- The cardinality of the complex numbers, as a set. -/
@[simp] lemma mk_univ_complex : #(set.univ : set ℂ) = 𝔠 :=
by rw [mk_univ, mk_complex]

/-- The complex numbers are not countable. -/
lemma not_countable_complex : ¬ countable (set.univ : set ℂ) :=
by { rw [← mk_set_le_omega, not_le, mk_univ_complex], apply cantor }

0 comments on commit 7967128

Please sign in to comment.