src/HOL/Multivariate_Analysis/Derivative.thy
changeset 61824 dcbe9f756ae0
parent 61810 3c5040d5694a
child 61880 ff4d33058566
--- a/src/HOL/Multivariate_Analysis/Derivative.thy	Mon Dec 07 10:49:08 2015 +0100
+++ b/src/HOL/Multivariate_Analysis/Derivative.thy	Thu Dec 10 13:38:40 2015 +0000
@@ -9,21 +9,6 @@
 imports Brouwer_Fixpoint Operator_Norm Uniform_Limit
 begin
 
-lemma netlimit_at_vector: (* TODO: move *)
-  fixes a :: "'a::real_normed_vector"
-  shows "netlimit (at a) = a"
-proof (cases "\<exists>x. x \<noteq> a")
-  case True then obtain x where x: "x \<noteq> a" ..
-  have "\<not> trivial_limit (at a)"
-    unfolding trivial_limit_def eventually_at dist_norm
-    apply clarsimp
-    apply (rule_tac x="a + scaleR (d / 2) (sgn (x - a))" in exI)
-    apply (simp add: norm_sgn sgn_zero_iff x)
-    done
-  then show ?thesis
-    by (rule netlimit_within [of a UNIV])
-qed simp
-
 declare has_derivative_bounded_linear[dest]
 
 subsection \<open>Derivatives\<close>