src/HOL/Old_Number_Theory/IntPrimes.thy
changeset 47163 248376f8881d
parent 47162 9d7d919b9fd8
child 49962 a8cc904a6820
--- a/src/HOL/Old_Number_Theory/IntPrimes.thy	Tue Mar 27 15:40:11 2012 +0200
+++ b/src/HOL/Old_Number_Theory/IntPrimes.thy	Tue Mar 27 15:53:48 2012 +0200
@@ -407,7 +407,7 @@
   apply (cut_tac a = a and n = n in zcong_lineq_ex, auto)
   apply (rule_tac x = "x * b mod n" in exI, safe)
     apply (simp_all (no_asm_simp))
-  apply (metis zcong_scalar zcong_zmod zmod_zmult1_eq mult_1 mult_assoc)
+  apply (metis zcong_scalar zcong_zmod mod_mult_right_eq mult_1 mult_assoc)
   done
 
 end