src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy
changeset 45031 9583f2b56f85
parent 44907 93943da0a010
child 47108 2a1953f0d20d
--- a/src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy	Tue Sep 20 15:23:17 2011 +0200
+++ b/src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy	Tue Sep 20 10:52:08 2011 -0700
@@ -1913,7 +1913,7 @@
 
 lemma has_derivative_at_dest_vec1:fixes f::"real\<Rightarrow>'a::real_normed_vector" shows
   "((f \<circ> dest_vec1) has_derivative (f' \<circ> dest_vec1)) (at (vec1 x)) = (f has_derivative f') (at x)"
-  using has_derivative_within_dest_vec1[where s=UNIV] by(auto simp add:within_UNIV)
+  using has_derivative_within_dest_vec1[where s=UNIV] by simp
 
 subsection {* In particular if we have a mapping into @{typ "real^1"}. *}