src/HOL/Analysis/Continuum_Not_Denumerable.thy
author blanchet
Mon, 25 Sep 2023 17:16:32 +0200
changeset 78694 5e995ceb7490
parent 77200 8f2e6186408f
permissions -rw-r--r--
allow (~) syntax in TPTP proofs for unapplied negation
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
63970
3b6a3632e754 HOL-Analysis: move Continuum_Not_Denumerable from Library
hoelzl
parents: 63881
diff changeset
     1
(*  Title:      HOL/Analysis/Continuum_Not_Denumerable.thy
56796
9f84219715a7 tuned proofs;
wenzelm
parents: 54797
diff changeset
     2
    Author:     Benjamin Porter, Monash University, NICTA, 2005
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
     3
    Author:     Johannes Hölzl, TU München
23461
wenzelm
parents: 23389
diff changeset
     4
*)
wenzelm
parents: 23389
diff changeset
     5
69517
dc20f278e8f3 tuned style and headers
nipkow
parents: 68607
diff changeset
     6
section \<open>Non-Denumerability of the Continuum\<close>
23461
wenzelm
parents: 23389
diff changeset
     7
63464
9d4dbb7a548a more standard name;
wenzelm
parents: 63092
diff changeset
     8
theory Continuum_Not_Denumerable
63970
3b6a3632e754 HOL-Analysis: move Continuum_Not_Denumerable from Library
hoelzl
parents: 63881
diff changeset
     9
imports
3b6a3632e754 HOL-Analysis: move Continuum_Not_Denumerable from Library
hoelzl
parents: 63881
diff changeset
    10
  Complex_Main 
66453
cc19f7ca2ed6 session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents: 63970
diff changeset
    11
  "HOL-Library.Countable_Set"
23461
wenzelm
parents: 23389
diff changeset
    12
begin
wenzelm
parents: 23389
diff changeset
    13
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69597
diff changeset
    14
subsection\<^marker>\<open>tag unimportant\<close> \<open>Abstract\<close>
23461
wenzelm
parents: 23389
diff changeset
    15
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    16
text \<open>
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    17
  The following document presents a proof that the Continuum is uncountable.
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    18
  It is formalised in the Isabelle/Isar theorem proving system.
23461
wenzelm
parents: 23389
diff changeset
    19
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    20
  \<^bold>\<open>Theorem:\<close> The Continuum \<open>\<real>\<close> is not denumerable. In other words, there does
63628
wenzelm
parents: 63540
diff changeset
    21
  not exist a function \<open>f: \<nat> \<Rightarrow> \<real>\<close> such that \<open>f\<close> is surjective.
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    22
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    23
  \<^bold>\<open>Outline:\<close> An elegant informal proof of this result uses Cantor's
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    24
  Diagonalisation argument. The proof presented here is not this one.
23461
wenzelm
parents: 23389
diff changeset
    25
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    26
  First we formalise some properties of closed intervals, then we prove the
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    27
  Nested Interval Property. This property relies on the completeness of the
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    28
  Real numbers and is the foundation for our argument. Informally it states
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    29
  that an intersection of countable closed intervals (where each successive
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    30
  interval is a subset of the last) is non-empty. We then assume a surjective
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    31
  function \<open>f: \<nat> \<Rightarrow> \<real>\<close> exists and find a real \<open>x\<close> such that \<open>x\<close> is not in the
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    32
  range of \<open>f\<close> by generating a sequence of closed intervals then using the
63628
wenzelm
parents: 63540
diff changeset
    33
  Nested Interval Property.
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    34
\<close>
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69597
diff changeset
    35
text\<^marker>\<open>tag important\<close> \<open>%whitespace\<close>
68607
67bb59e49834 make theorem, corollary, and proposition %important for HOL-Analysis manual
immler
parents: 67968
diff changeset
    36
theorem real_non_denum: "\<nexists>f :: nat \<Rightarrow> real. surj f"
67bb59e49834 make theorem, corollary, and proposition %important for HOL-Analysis manual
immler
parents: 67968
diff changeset
    37
proof
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    38
  assume "\<exists>f::nat \<Rightarrow> real. surj f"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    39
  then obtain f :: "nat \<Rightarrow> real" where "surj f" ..
56796
9f84219715a7 tuned proofs;
wenzelm
parents: 54797
diff changeset
    40
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 69565
diff changeset
    41
  txt \<open>First we construct a sequence of nested intervals, ignoring \<^term>\<open>range f\<close>.\<close>
23461
wenzelm
parents: 23389
diff changeset
    42
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    43
  have "a < b \<Longrightarrow> \<exists>ka kb. ka < kb \<and> {ka..kb} \<subseteq> {a..b} \<and> c \<notin> {ka..kb}" for a b c :: real
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    44
    by (auto simp add: not_le cong: conj_cong)
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    45
      (metis dense le_less_linear less_linear less_trans order_refl)
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    46
  then obtain i j where ij:
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    47
    "a < b \<Longrightarrow> i a b c < j a b c"
63060
293ede07b775 some uses of 'obtain' with structure statement;
wenzelm
parents: 63040
diff changeset
    48
      "a < b \<Longrightarrow> {i a b c .. j a b c} \<subseteq> {a .. b}"
293ede07b775 some uses of 'obtain' with structure statement;
wenzelm
parents: 63040
diff changeset
    49
      "a < b \<Longrightarrow> c \<notin> {i a b c .. j a b c}"
293ede07b775 some uses of 'obtain' with structure statement;
wenzelm
parents: 63040
diff changeset
    50
    for a b c :: real
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    51
    by metis
23461
wenzelm
parents: 23389
diff changeset
    52
63040
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 62083
diff changeset
    53
  define ivl where "ivl =
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 62083
diff changeset
    54
    rec_nat (f 0 + 1, f 0 + 2) (\<lambda>n x. (i (fst x) (snd x) (f n), j (fst x) (snd x) (f n)))"
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 62083
diff changeset
    55
  define I where "I n = {fst (ivl n) .. snd (ivl n)}" for n
23461
wenzelm
parents: 23389
diff changeset
    56
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    57
  have ivl [simp]:
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    58
    "ivl 0 = (f 0 + 1, f 0 + 2)"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    59
    "\<And>n. ivl (Suc n) = (i (fst (ivl n)) (snd (ivl n)) (f n), j (fst (ivl n)) (snd (ivl n)) (f n))"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    60
    unfolding ivl_def by simp_all
56796
9f84219715a7 tuned proofs;
wenzelm
parents: 54797
diff changeset
    61
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 60308
diff changeset
    62
  txt \<open>This is a decreasing sequence of non-empty intervals.\<close>
23461
wenzelm
parents: 23389
diff changeset
    63
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    64
  have less: "fst (ivl n) < snd (ivl n)" for n
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    65
    by (induct n) (auto intro!: ij)
23461
wenzelm
parents: 23389
diff changeset
    66
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    67
  have "decseq I"
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    68
    unfolding I_def decseq_Suc_iff ivl fst_conv snd_conv
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    69
    by (intro ij allI less)
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    70
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 60308
diff changeset
    71
  txt \<open>Now we apply the finite intersection property of compact sets.\<close>
23461
wenzelm
parents: 23389
diff changeset
    72
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    73
  have "I 0 \<inter> (\<Inter>i. I i) \<noteq> {}"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    74
  proof (rule compact_imp_fip_image)
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    75
    fix S :: "nat set"
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    76
    assume fin: "finite S"
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    77
    have "{} \<subset> I (Max (insert 0 S))"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    78
      unfolding I_def using less[of "Max (insert 0 S)"] by auto
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    79
    also have "I (Max (insert 0 S)) \<subseteq> (\<Inter>i\<in>insert 0 S. I i)"
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    80
      using fin decseqD[OF \<open>decseq I\<close>, of _ "Max (insert 0 S)"]
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    81
      by (auto simp: Max_ge_iff)
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    82
    also have "(\<Inter>i\<in>insert 0 S. I i) = I 0 \<inter> (\<Inter>i\<in>S. I i)"
56796
9f84219715a7 tuned proofs;
wenzelm
parents: 54797
diff changeset
    83
      by auto
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    84
    finally show "I 0 \<inter> (\<Inter>i\<in>S. I i) \<noteq> {}"
53372
f5a6313c7fe4 tuned proof;
wenzelm
parents: 40702
diff changeset
    85
      by auto
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    86
  qed (auto simp: I_def)
63060
293ede07b775 some uses of 'obtain' with structure statement;
wenzelm
parents: 63040
diff changeset
    87
  then obtain x where "x \<in> I n" for n
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    88
    by blast
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 60308
diff changeset
    89
  moreover from \<open>surj f\<close> obtain j where "x = f j"
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    90
    by blast
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    91
  ultimately have "f j \<in> I (Suc j)"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    92
    by blast
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    93
  with ij(3)[OF less] show False
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    94
    unfolding I_def ivl fst_conv snd_conv by auto
23461
wenzelm
parents: 23389
diff changeset
    95
qed
wenzelm
parents: 23389
diff changeset
    96
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
    97
lemma uncountable_UNIV_real: "uncountable (UNIV :: real set)"
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
    98
  using real_non_denum unfolding uncountable_def by auto
23461
wenzelm
parents: 23389
diff changeset
    99
75078
ec86cb2418e1 an assortment of new or stronger lemmas
paulson <lp15@cam.ac.uk>
parents: 70136
diff changeset
   100
corollary complex_non_denum: "\<nexists>f :: nat \<Rightarrow> complex. surj f"
ec86cb2418e1 an assortment of new or stronger lemmas
paulson <lp15@cam.ac.uk>
parents: 70136
diff changeset
   101
  by (metis (full_types) Re_complex_of_real comp_surj real_non_denum surj_def)
ec86cb2418e1 an assortment of new or stronger lemmas
paulson <lp15@cam.ac.uk>
parents: 70136
diff changeset
   102
ec86cb2418e1 an assortment of new or stronger lemmas
paulson <lp15@cam.ac.uk>
parents: 70136
diff changeset
   103
lemma uncountable_UNIV_complex: "uncountable (UNIV :: complex set)"
ec86cb2418e1 an assortment of new or stronger lemmas
paulson <lp15@cam.ac.uk>
parents: 70136
diff changeset
   104
  using complex_non_denum unfolding uncountable_def by auto
ec86cb2418e1 an assortment of new or stronger lemmas
paulson <lp15@cam.ac.uk>
parents: 70136
diff changeset
   105
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   106
lemma bij_betw_open_intervals:
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   107
  fixes a b c d :: real
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   108
  assumes "a < b" "c < d"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   109
  shows "\<exists>f. bij_betw f {a<..<b} {c<..<d}"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   110
proof -
63040
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 62083
diff changeset
   111
  define f where "f a b c d x = (d - c)/(b - a) * (x - a) + c" for a b c d x :: real
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   112
  {
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   113
    fix a b c d x :: real
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   114
    assume *: "a < b" "c < d" "a < x" "x < b"
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   115
    moreover from * have "(d - c) * (x - a) < (d - c) * (b - a)"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   116
      by (intro mult_strict_left_mono) simp_all
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   117
    moreover from * have "0 < (d - c) * (x - a) / (b - a)"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   118
      by simp
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   119
    ultimately have "f a b c d x < d" "c < f a b c d x"
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   120
      by (simp_all add: f_def field_simps)
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   121
  }
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   122
  with assms have "bij_betw (f a b c d) {a<..<b} {c<..<d}"
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   123
    by (intro bij_betw_byWitness[where f'="f c d a b"]) (auto simp: f_def)
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   124
  then show ?thesis by auto
23461
wenzelm
parents: 23389
diff changeset
   125
qed
wenzelm
parents: 23389
diff changeset
   126
57234
596a499318ab clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
hoelzl
parents: 56796
diff changeset
   127
lemma bij_betw_tan: "bij_betw tan {-pi/2<..<pi/2} UNIV"
59872
db4000b71fdb Theorem "arctan" is no longer a default simprule
paulson <lp15@cam.ac.uk>
parents: 59720
diff changeset
   128
  using arctan_ubound by (intro bij_betw_byWitness[where f'=arctan]) (auto simp: arctan arctan_tan)
23461
wenzelm
parents: 23389
diff changeset
   129
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   130
lemma uncountable_open_interval: "uncountable {a<..<b} \<longleftrightarrow> a < b" for a b :: real
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   131
proof
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   132
  show "a < b" if "uncountable {a<..<b}"
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   133
    using uncountable_def that by force
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   134
  show "uncountable {a<..<b}" if "a < b"
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   135
  proof -
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   136
    obtain f where "bij_betw f {a <..< b} {-pi/2<..<pi/2}"
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 60308
diff changeset
   137
      using bij_betw_open_intervals[OF \<open>a < b\<close>, of "-pi/2" "pi/2"] by auto
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   138
    then show ?thesis
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   139
      by (metis bij_betw_tan uncountable_bij_betw uncountable_UNIV_real)
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   140
  qed
23461
wenzelm
parents: 23389
diff changeset
   141
qed
wenzelm
parents: 23389
diff changeset
   142
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   143
lemma uncountable_half_open_interval_1: "uncountable {a..<b} \<longleftrightarrow> a < b" for a b :: real
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   144
  apply auto
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   145
  using atLeastLessThan_empty_iff
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   146
  apply fastforce
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   147
  using uncountable_open_interval [of a b]
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   148
  apply (metis countable_Un_iff ivl_disj_un_singleton(3))
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   149
  done
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   150
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   151
lemma uncountable_half_open_interval_2: "uncountable {a<..b} \<longleftrightarrow> a < b" for a b :: real
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   152
  apply auto
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   153
  using atLeastLessThan_empty_iff
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   154
  apply fastforce
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   155
  using uncountable_open_interval [of a b]
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   156
  apply (metis countable_Un_iff ivl_disj_un_singleton(4))
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   157
  done
60308
f7e406aba90d uncountability: open interval equivalences
paulson <lp15@cam.ac.uk>
parents: 59872
diff changeset
   158
61880
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   159
lemma real_interval_avoid_countable_set:
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   160
  fixes a b :: real and A :: "real set"
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   161
  assumes "a < b" and "countable A"
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   162
  shows "\<exists>x\<in>{a<..<b}. x \<notin> A"
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   163
proof -
63540
f8652d0534fa tuned proofs -- avoid unstructured calculation;
wenzelm
parents: 63465
diff changeset
   164
  from \<open>countable A\<close> have *: "countable (A \<inter> {a<..<b})"
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   165
    by auto
63540
f8652d0534fa tuned proofs -- avoid unstructured calculation;
wenzelm
parents: 63465
diff changeset
   166
  with \<open>a < b\<close> have "\<not> countable {a<..<b}"
61880
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   167
    by (simp add: uncountable_open_interval)
63540
f8652d0534fa tuned proofs -- avoid unstructured calculation;
wenzelm
parents: 63465
diff changeset
   168
  with * have "A \<inter> {a<..<b} \<noteq> {a<..<b}"
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   169
    by auto
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   170
  then have "A \<inter> {a<..<b} \<subset> {a<..<b}"
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   171
    by (intro psubsetI) auto
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   172
  then have "\<exists>x. x \<in> {a<..<b} - A \<inter> {a<..<b}"
61880
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   173
    by (rule psubset_imp_ex_mem)
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   174
  then show ?thesis
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   175
    by auto
61880
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   176
qed
ff4d33058566 moved some theorems from the CLT proof; reordered some theorems / notation
hoelzl
parents: 61585
diff changeset
   177
63881
b746b19197bd lots of new results about topology, affine dimension etc
paulson <lp15@cam.ac.uk>
parents: 63628
diff changeset
   178
lemma uncountable_closed_interval: "uncountable {a..b} \<longleftrightarrow> a < b" for a b :: real
77200
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 75078
diff changeset
   179
  using infinite_Icc_iff by (fastforce dest: countable_finite real_interval_avoid_countable_set)
63881
b746b19197bd lots of new results about topology, affine dimension etc
paulson <lp15@cam.ac.uk>
parents: 63628
diff changeset
   180
62083
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   181
lemma open_minus_countable:
63465
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   182
  fixes S A :: "real set"
d7610beb98bc misc tuning and modernization;
wenzelm
parents: 63464
diff changeset
   183
  assumes "countable A" "S \<noteq> {}" "open S"
62083
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   184
  shows "\<exists>x\<in>S. x \<notin> A"
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   185
proof -
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   186
  obtain x where "x \<in> S"
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   187
    using \<open>S \<noteq> {}\<close> by auto
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   188
  then obtain e where "0 < e" "{y. dist y x < e} \<subseteq> S"
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   189
    using \<open>open S\<close> by (auto simp: open_dist subset_eq)
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   190
  moreover have "{y. dist y x < e} = {x - e <..< x + e}"
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   191
    by (auto simp: dist_real_def)
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   192
  ultimately have "uncountable (S - A)"
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   193
    using uncountable_open_interval[of "x - e" "x + e"] \<open>countable A\<close>
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   194
    by (intro uncountable_minus_countable) (auto dest: countable_subset)
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   195
  then show ?thesis
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   196
    unfolding uncountable_def by auto
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   197
qed
7582b39f51ed add the proof of the central limit theorem
hoelzl
parents: 61975
diff changeset
   198
23461
wenzelm
parents: 23389
diff changeset
   199
end