src/HOL/ex/ThreeDivides.thy
changeset 57512 cc97b347b301
parent 41413 64cd30d6b0b8
child 57514 bdc2c6b40bf2
--- a/src/HOL/ex/ThreeDivides.thy	Fri Jul 04 20:07:08 2014 +0200
+++ b/src/HOL/ex/ThreeDivides.thy	Fri Jul 04 20:18:47 2014 +0200
@@ -88,7 +88,7 @@
 lemma three_divs_1:
   fixes D :: "nat \<Rightarrow> nat"
   shows "3 dvd (\<Sum>x<nd. D x * (10^x - 1))"
-  by (subst nat_mult_commute, rule div_sum) (simp add: three_divs_0 [simplified])
+  by (subst mult.commute, rule div_sum) (simp add: three_divs_0 [simplified])
 
 text {* Using lemmas @{text "digit_diff_split"} and 
 @{text "three_divs_1"} we now prove the following lemma.