src/HOL/Real/HahnBanach/HahnBanach.thy
changeset 8902 a705822f4e2a
parent 8838 4eaa99f0d223
child 9013 9dd0274f76af
--- a/src/HOL/Real/HahnBanach/HahnBanach.thy	Sun May 21 14:44:01 2000 +0200
+++ b/src/HOL/Real/HahnBanach/HahnBanach.thy	Sun May 21 14:49:28 2000 +0200
@@ -48,7 +48,7 @@
 txt {* Define $M$ as the set of all norm-preserving extensions of $F$.  *};
 
   def M == "norm_pres_extensions E p F f";
-  {{;
+  {;
     fix c; assume "c : chain M" "EX x. x:c";
 
 txt {* Show that every non-empty chain $c$ in $M$ has an upper bound in $M$: $\Union c$ is greater that every element of the chain $c$, so $\Union c$ is an upper bound of $c$ that lies in $M$. *};
@@ -82,7 +82,7 @@
           by (rule sup_norm_pres [OF _ _ a]) (simp!)+;
       qed;
     qed;
-  }};
+  };
   
 txt {* With Zorn's Lemma we can conclude that there is a maximal element $g$ in $M$. *};
 
@@ -340,7 +340,7 @@
   It is even the least upper bound, because every upper bound of $M$
   is also an upper bound for $\Union c$, as $\Union c\in M$) *};
 
-  {{;
+  {;
     fix c; assume "c:chain M" "EX x. x:c";
     have "Union c : M";
 
@@ -372,7 +372,7 @@
           by (rule sup_norm_pres, rule a) (simp!)+;
       qed;
     qed;
-  }};
+  };
  
   txt {* According to Zorn's Lemma there is
   a maximal norm-preserving extension $g\in M$. *};