src/HOL/Deriv.thy
changeset 63170 eae6549dbea2
parent 63092 a949b2a5f51d
child 63263 c6c95d64607a
--- a/src/HOL/Deriv.thy	Fri May 27 20:13:06 2016 +0200
+++ b/src/HOL/Deriv.thy	Fri May 27 20:23:55 2016 +0200
@@ -857,7 +857,7 @@
 lemma DERIV_chain': "(f has_field_derivative D) (at x within s) \<Longrightarrow> DERIV g (f x) :> E \<Longrightarrow> 
   ((\<lambda>x. g (f x)) has_field_derivative E * D) (at x within s)"
   using has_derivative_compose[of f "op * D" x s g "op * E"]
-  unfolding has_field_derivative_def mult_commute_abs ac_simps .
+  by (simp only: has_field_derivative_def mult_commute_abs ac_simps)
 
 corollary DERIV_chain2: "DERIV f (g x) :> Da \<Longrightarrow> (g has_field_derivative Db) (at x within s) \<Longrightarrow>
   ((\<lambda>x. f (g x)) has_field_derivative Da * Db) (at x within s)"