src/HOL/Algebra/IntRing.thy
changeset 57512 cc97b347b301
parent 55991 3fa6e6c81788
child 57514 bdc2c6b40bf2
--- a/src/HOL/Algebra/IntRing.thy	Fri Jul 04 20:07:08 2014 +0200
+++ b/src/HOL/Algebra/IntRing.thy	Fri Jul 04 20:18:47 2014 +0200
@@ -271,11 +271,11 @@
   then have "p dvd a \<or> p dvd b"
     by (metis prime prime_dvd_mult_eq_int)
   then show "(\<exists>x. a = x * int p) \<or> (\<exists>x. b = x * int p)"
-    by (metis dvd_def mult_commute)
+    by (metis dvd_def mult.commute)
 next
   assume "UNIV = {uu. EX x. uu = x * int p}"
   then obtain x where "1 = x * int p" by best
-  then have "\<bar>int p * x\<bar> = 1" by (simp add: mult_commute)
+  then have "\<bar>int p * x\<bar> = 1" by (simp add: mult.commute)
   then show False
     by (metis abs_of_nat int_1 of_nat_eq_iff abs_zmult_eq_1 one_not_prime_nat prime)
 qed