src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy
changeset 34999 5312d2ffee3b
parent 34964 4e8be3c04d37
child 35028 108662d50512
--- a/src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy	Thu Feb 04 13:36:52 2010 +0100
+++ b/src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy	Thu Feb 04 14:45:08 2010 +0100
@@ -5906,7 +5906,7 @@
       using c and zero_le_dist[of x y] by auto
     hence "y = x" by auto
   }
-  ultimately show ?thesis unfolding Bex1_def using `x\<in>s` by blast+
+  ultimately show ?thesis using `x\<in>s` by blast+
 qed
 
 subsection{* Edelstein fixed point theorem.                                            *}
@@ -5923,7 +5923,7 @@
     hence "x = y" using `x\<in>s` and dist[THEN bspec[where x=x], THEN bspec[where x=y]]
       unfolding g[THEN bspec[where x=x], OF `x\<in>s`]
       unfolding g[THEN bspec[where x=y], OF `y\<in>s`] by auto  }
-  thus ?thesis unfolding Bex1_def using `x\<in>s` and g by blast+
+  thus ?thesis using `x\<in>s` and g by blast+
 next
   case True
   then obtain x where [simp]:"x\<in>s" and "g x \<noteq> x" by auto
@@ -6028,7 +6028,7 @@
   { fix x assume "x\<in>s" "g x = x" "x\<noteq>a"
     hence "False" using dist[THEN bspec[where x=a], THEN bspec[where x=x]]
       using `g a = a` and `a\<in>s` by auto  }
-  ultimately show "\<exists>!x\<in>s. g x = x" unfolding Bex1_def using `a\<in>s` by blast
+  ultimately show "\<exists>!x\<in>s. g x = x" using `a\<in>s` by blast
 qed
 
 end