src/HOL/ex/Gauge_Integration.thy
changeset 57512 cc97b347b301
parent 56541 0e3abadbef39
child 58247 98d0f85d247f
--- a/src/HOL/ex/Gauge_Integration.thy	Fri Jul 04 20:07:08 2014 +0200
+++ b/src/HOL/ex/Gauge_Integration.thy	Fri Jul 04 20:18:47 2014 +0200
@@ -510,9 +510,9 @@
 next
   case False
   then have "inverse (z - x) * (f z - f x - f' x * (z - x)) = (f z - f x) / (z - x) - f' x"
-    apply (subst mult_commute)
+    apply (subst mult.commute)
     apply (simp add: left_diff_distrib)
-    apply (simp add: mult_assoc divide_inverse)
+    apply (simp add: mult.assoc divide_inverse)
     apply (simp add: ring_distribs)
     done
   moreover from False `\<bar>z - x\<bar> < s` have "\<bar>(f z - f x) / (z - x) - f' x\<bar> < e / 2"