src/HOL/Deriv.thy
changeset 57418 6ab1c7cb0b8d
parent 56541 0e3abadbef39
child 57512 cc97b347b301
--- a/src/HOL/Deriv.thy	Fri Jun 27 22:08:55 2014 +0200
+++ b/src/HOL/Deriv.thy	Sat Jun 28 09:16:42 2014 +0200
@@ -357,7 +357,7 @@
     have "((\<lambda>x. f i x * (\<Prod>i\<in>I. f i x)) has_derivative ?P) (at x within s)"
       using insert by (intro has_derivative_mult) auto
     also have "?P = (\<lambda>y. \<Sum>i'\<in>insert i I. f' i' y * (\<Prod>j\<in>insert i I - {i'}. f j x))"
-      using insert(1,2) by (auto simp add: setsum_right_distrib insert_Diff_if intro!: ext setsum_cong)
+      using insert(1,2) by (auto simp add: setsum_right_distrib insert_Diff_if intro!: ext setsum.cong)
     finally show ?case
       using insert by simp
   qed simp