src/HOL/Number_Theory/Eratosthenes.thy
changeset 64243 aee949f6642d
parent 63633 2accfb71e33b
child 65417 fc41a5650fb1
--- a/src/HOL/Number_Theory/Eratosthenes.thy	Sun Oct 16 09:31:05 2016 +0200
+++ b/src/HOL/Number_Theory/Eratosthenes.thy	Sun Oct 16 09:31:05 2016 +0200
@@ -143,7 +143,7 @@
       then have "u + (w - u mod w) = w + (u - u mod w)"
         by simp
       then have "u + (w - u mod w) = w + u div w * w"
-        by (simp add: div_mod_equality' [symmetric])
+        by (simp add: minus_mod_eq_div_mult)
     }
     then have "w dvd v + w + r + (w - v mod w) \<longleftrightarrow> w dvd m + w + r + (w - m mod w)"
       by (simp add: add.assoc add.left_commute [of m] add.left_commute [of v]