src/HOL/Analysis/Interval_Integral.thy
changeset 70613 8b7f6ecb3369
parent 70365 4df0628e8545
child 71827 5e315defb038
--- a/src/HOL/Analysis/Interval_Integral.thy	Tue Aug 27 13:22:33 2019 +0200
+++ b/src/HOL/Analysis/Interval_Integral.thy	Tue Aug 27 16:25:00 2019 +0200
@@ -8,10 +8,6 @@
   imports Equivalence_Lebesgue_Henstock_Integration
 begin
 
-lemma continuous_on_vector_derivative:
-  "(\<And>x. x \<in> S \<Longrightarrow> (f has_vector_derivative f' x) (at x within S)) \<Longrightarrow> continuous_on S f"
-  by (auto simp: continuous_on_eq_continuous_within intro!: has_vector_derivative_continuous)
-
 definition "einterval a b = {x. a < ereal x \<and> ereal x < b}"
 
 lemma einterval_eq[simp]: