src/Doc/Demo_Easychair/Document.thy
author haftmann
Thu, 19 Jun 2025 17:15:40 +0200
changeset 82734 89347c0cc6a3
parent 76987 4c275405faae
permissions -rw-r--r--
treat map_filter similar to list_all, list_ex, list_ex1
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
76396
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     1
theory Document
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     2
  imports Main
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     3
begin
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     4
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     5
section \<open>Some section\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     6
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     7
subsection \<open>Some subsection\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     8
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
     9
subsection \<open>Some subsubsection\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    10
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    11
subsubsection \<open>Some subsubsubsection\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    12
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    13
paragraph \<open>A paragraph.\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    14
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    15
text \<open>Informal bla bla.\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    16
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    17
definition "foo = True"  \<comment> \<open>side remark on \<^const>\<open>foo\<close>\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    18
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    19
definition "bar = False"  \<comment> \<open>side remark on \<^const>\<open>bar\<close>\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    20
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    21
lemma foo unfolding foo_def ..
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    22
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    23
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    24
paragraph \<open>Another paragraph.\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    25
76987
4c275405faae isabelle update -u cite;
wenzelm
parents: 76396
diff changeset
    26
text \<open>See also \<^cite>\<open>\<open>\S3\<close> in "isabelle-system"\<close>.\<close>
76396
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    27
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    28
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    29
section \<open>Formal proof of Cantor's theorem\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    30
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    31
text_raw \<open>\isakeeptag{proof}\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    32
text \<open>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    33
  Cantor's Theorem states that there is no surjection from
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    34
  a set to its powerset.  The proof works by diagonalization.  E.g.\ see
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    35
  \<^item> \<^url>\<open>http://mathworld.wolfram.com/CantorDiagonalMethod.html\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    36
  \<^item> \<^url>\<open>https://en.wikipedia.org/wiki/Cantor's_diagonal_argument\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    37
\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    38
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    39
theorem Cantor: "\<nexists>f :: 'a \<Rightarrow> 'a set. \<forall>A. \<exists>x. A = f x"
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    40
proof
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    41
  assume "\<exists>f :: 'a \<Rightarrow> 'a set. \<forall>A. \<exists>x. A = f x"
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    42
  then obtain f :: "'a \<Rightarrow> 'a set" where *: "\<forall>A. \<exists>x. A = f x" ..
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    43
  let ?D = "{x. x \<notin> f x}"
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    44
  from * obtain a where "?D = f a" by blast
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    45
  moreover have "a \<in> ?D \<longleftrightarrow> a \<notin> f a" by blast
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    46
  ultimately show False by blast
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    47
qed
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    48
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    49
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    50
subsection \<open>Lorem ipsum dolor\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    51
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    52
text \<open>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    53
  Lorem ipsum dolor sit amet, consectetur adipiscing elit. Donec id ipsum
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    54
  sapien. Vivamus malesuada enim nibh, a tristique nisi sodales ac. Praesent
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    55
  ut sem consectetur, interdum tellus ac, sodales nulla. Quisque vel diam at
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    56
  risus tempus tempor eget a tortor. Suspendisse potenti. Nulla erat lacus,
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    57
  dignissim sed volutpat nec, feugiat non leo. Nunc blandit et justo sed
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    58
  venenatis. Donec scelerisque placerat magna, et congue nulla convallis vel.
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    59
  Cras tristique dolor consequat dolor tristique rutrum. Suspendisse ultrices
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    60
  sem nibh, et suscipit felis ultricies at. Aliquam venenatis est vel nulla
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    61
  efficitur ornare. Lorem ipsum dolor sit amet, consectetur adipiscing elit.
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    62
\<close>
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    63
389d77e6be9f support for Easychair style with demo document;
wenzelm
parents:
diff changeset
    64
end