merged
authorwenzelm
Thu, 20 Mar 2014 23:38:34 +0100
changeset 56236 713ae0c9e652
parent 56227 67a5f004583d (diff)
parent 56235 083b41092afe (current diff)
child 56237 69a9dfe71aed
merged
--- a/src/HOL/Multivariate_Analysis/Derivative.thy	Thu Mar 20 23:13:33 2014 +0100
+++ b/src/HOL/Multivariate_Analysis/Derivative.thy	Thu Mar 20 23:38:34 2014 +0100
@@ -888,7 +888,7 @@
 text {* In particular. *}
 
 lemma has_derivative_zero_constant:
-  fixes f :: "real \<Rightarrow> real"
+  fixes f :: "'a::real_normed_vector \<Rightarrow> 'b::real_inner"
   assumes "convex s"
     and "\<forall>x\<in>s. (f has_derivative (\<lambda>h. 0)) (at x within s)"
   shows "\<exists>c. \<forall>x\<in>s. f x = c"
@@ -914,7 +914,7 @@
 qed
 
 lemma has_derivative_zero_unique:
-  fixes f :: "real \<Rightarrow> real"
+  fixes f :: "'a::real_normed_vector \<Rightarrow> 'b::real_inner"
   assumes "convex s"
     and "a \<in> s"
     and "f a = c"
@@ -1184,7 +1184,7 @@
 text {* See Sussmann: "Multidifferential calculus", Theorem 2.1.1 *}
 
 lemma sussmann_open_mapping:
-  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
+  fixes f :: "'a::real_normed_vector \<Rightarrow> 'b::euclidean_space"
   assumes "open s"
     and "continuous_on s f"
     and "x \<in> s"