src/HOL/Real/HahnBanach/ZornLemma.thy
author wenzelm
Mon, 21 Feb 2000 14:10:21 +0100
changeset 8272 1329173b56ed
parent 8104 d9b3a224c0e6
child 8280 259073d16f84
permissions -rw-r--r--
tuned footnote;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     1
(*  Title:      HOL/Real/HahnBanach/ZornLemma.thy
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     2
    ID:         $Id$
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     3
    Author:     Gertrud Bauer, TU Munich
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     4
*)
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     5
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     6
header {* Zorn's Lemma *};
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     7
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     8
theory ZornLemma = Aux + Zorn:;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
     9
8104
wenzelm
parents: 7978
diff changeset
    10
text {* Zorn's Lemmas states: if every linear ordered subset of an
wenzelm
parents: 7978
diff changeset
    11
ordered set $S$ has an upper bound in $S$, then there exists a maximal
wenzelm
parents: 7978
diff changeset
    12
element in $S$.  In our application, $S$ is a set of sets ordered by
wenzelm
parents: 7978
diff changeset
    13
set inclusion. Since the union of a chain of sets is an upper bound
wenzelm
parents: 7978
diff changeset
    14
for all elements of the chain, the conditions of Zorn's lemma can be
wenzelm
parents: 7978
diff changeset
    15
modified: if $S$ is non-empty, it suffices to show that for every
wenzelm
parents: 7978
diff changeset
    16
non-empty chain $c$ in $S$ the union of $c$ also lies in $S$. *};
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    17
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    18
theorem Zorn's_Lemma: 
8104
wenzelm
parents: 7978
diff changeset
    19
  "(!!c. c: chain S ==> EX x. x:c ==> Union c : S) ==> a:S
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    20
  ==>  EX y: S. ALL z: S. y <= z --> y = z";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    21
proof (rule Zorn_Lemma2);
8104
wenzelm
parents: 7978
diff changeset
    22
  txt_raw {* \footnote{See
8272
1329173b56ed tuned footnote;
wenzelm
parents: 8104
diff changeset
    23
  \url{http://isabelle.in.tum.de/library/HOL/HOL-Real/Zorn.html}} \isanewline *};
8104
wenzelm
parents: 7978
diff changeset
    24
  assume r: "!!c. c: chain S ==> EX x. x:c ==> Union c : S";
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    25
  assume aS: "a:S";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    26
  show "ALL c:chain S. EX y:S. ALL z:c. z <= y";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    27
  proof;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    28
    fix c; assume "c:chain S"; 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    29
    show "EX y:S. ALL z:c. z <= y";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    30
    proof (rule case_split);
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    31
 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    32
      txt{* If $c$ is an empty chain, then every element
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    33
      in $S$ is an upper bound of $c$. *};
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    34
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    35
      assume "c={}"; 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    36
      with aS; show ?thesis; by fast;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    37
7927
b50446a33c16 update by Gertrud Bauer;
wenzelm
parents: 7917
diff changeset
    38
      txt{* If $c$ is non-empty, then $\Union c$ 
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    39
      is an upper bound of $c$, lying in $S$. *};
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    40
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    41
    next;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    42
      assume c: "c~={}";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    43
      show ?thesis; 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    44
      proof; 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    45
        show "ALL z:c. z <= Union c"; by fast;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    46
        show "Union c : S"; 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    47
        proof (rule r);
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    48
          from c; show "EX x. x:c"; by fast;  
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    49
        qed;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    50
      qed;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    51
    qed;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    52
  qed;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    53
qed;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    54
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents:
diff changeset
    55
end;