# HG changeset patch # User wenzelm # Date 947101634 -3600 # Node ID 284d6a3c8bd2b5fc22146816aae48ab8faeff8bb # Parent de9fae0cdfdebff622cd7a8b51ea480636b51d6c oops; diff -r de9fae0cdfde -r 284d6a3c8bd2 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$. *};