src/HOL/Real/HahnBanach/Zorn_Lemma.thy
author wenzelm
Fri, 10 Sep 1999 17:28:51 +0200
changeset 7535 599d3414b51d
child 7566 c5a3f980a7af
permissions -rw-r--r--
The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar) (by Gertrud Bauer, TU Munich);


theory Zorn_Lemma = Zorn:;


lemma Zorn's_Lemma: "a:S ==> (!!c. c: chain S ==> EX x. x:c ==> Union c : S) ==>
 EX y: S. ALL z: S. y <= z --> y = z";
proof (rule Zorn_Lemma2);
  assume aS: "a:S";
  assume r: "!!c. c: chain S ==> EX x. x:c ==> Union c : S";
  show "ALL c:chain S. EX y:S. ALL z:c. z <= y";
  proof;
    fix c; assume "c:chain S"; 
    have s: "EX x. x:c ==> Union c : S";
      by (rule r);
    show "EX y:S. ALL z:c. z <= y";
    proof (rule case [of "c={}"]);
      assume "c={}"; 
      show ?thesis; by fast;
    next;
      assume "c~={}";
      show ?thesis; 
      proof;
        have "EX x. x:c"; by fast;
        thus "Union c : S"; by (rule s);
        show "ALL z:c. z <= Union c"; by fast;
      qed;
    qed;
  qed;
qed;



end;