src/HOL/Real/HahnBanach/ZornLemma.thy
changeset 8272 1329173b56ed
parent 8104 d9b3a224c0e6
child 8280 259073d16f84
     1.1 --- a/src/HOL/Real/HahnBanach/ZornLemma.thy	Mon Feb 21 14:09:40 2000 +0100
     1.2 +++ b/src/HOL/Real/HahnBanach/ZornLemma.thy	Mon Feb 21 14:10:21 2000 +0100
     1.3 @@ -20,7 +20,7 @@
     1.4    ==>  EX y: S. ALL z: S. y <= z --> y = z";
     1.5  proof (rule Zorn_Lemma2);
     1.6    txt_raw {* \footnote{See
     1.7 -  \url{http://isabelle.in.tum.de/library/HOL/HOL-Real/Zorn.html}}*};
     1.8 +  \url{http://isabelle.in.tum.de/library/HOL/HOL-Real/Zorn.html}} \isanewline *};
     1.9    assume r: "!!c. c: chain S ==> EX x. x:c ==> Union c : S";
    1.10    assume aS: "a:S";
    1.11    show "ALL c:chain S. EX y:S. ALL z:c. z <= y";