oops;
authorwenzelm
Wed, 05 Jan 2000 20:47:14 +0100
changeset 8107 284d6a3c8bd2
parent 8106 de9fae0cdfde
child 8108 ce4bb031d664
oops;
src/HOL/Real/HahnBanach/HahnBanach.thy
--- a/src/HOL/Real/HahnBanach/HahnBanach.thy	Wed Jan 05 18:27:07 2000 +0100
+++ b/src/HOL/Real/HahnBanach/HahnBanach.thy	Wed Jan 05 20:47:14 2000 +0100
@@ -117,7 +117,7 @@
           & is_subspace H E & is_subspace F H
           & graph F f <= graph H h
           & (ALL x:H. h x <= p x)"; by (simp! add: norm_pres_extension_D);
-        thus ?thesis; by blast;
+        thus ?thesis; by (elim exE conjE) rule;
       qed;
       have h: "is_vectorspace H"; ..;
 
@@ -185,7 +185,7 @@
                 thus "- p (u + x0) - h u <= p (v + x0) - h v";
                   by (rule real_diff_ineq_swap);
               qed;
-              thus ?thesis; by blast;
+              thus ?thesis; by rule rule;
             qed;
 
 txt {* Define the extension $h_0$ of $h$ to $H_0$ using $\xi$.  *};