src/HOL/Multivariate_Analysis/Derivative.thy
changeset 51733 70abecafe9ac
parent 51642 400ec5ae7f8f
child 53077 a1b3784f8129
--- a/src/HOL/Multivariate_Analysis/Derivative.thy	Mon Apr 22 16:36:02 2013 +0200
+++ b/src/HOL/Multivariate_Analysis/Derivative.thy	Mon Apr 22 18:39:12 2013 +0200
@@ -1433,7 +1433,6 @@
 qed
 
 lemma vector_derivative_unique_within_closed_interval:
-  fixes f::"real \<Rightarrow> 'n::ordered_euclidean_space"
   assumes "a < b" and "x \<in> {a..b}"
   assumes "(f has_vector_derivative f') (at x within {a..b})"
   assumes "(f has_vector_derivative f'') (at x within {a..b})"
@@ -1460,7 +1459,6 @@
   unfolding has_vector_derivative_def by auto
 
 lemma vector_derivative_within_closed_interval:
-  fixes f::"real \<Rightarrow> 'a::ordered_euclidean_space"
   assumes "a < b" and "x \<in> {a..b}"
   assumes "(f has_vector_derivative f') (at x within {a..b})"
   shows "vector_derivative f (at x within {a..b}) = f'"