src/HOL/Quotient_Examples/Quotient_Int.thy
changeset 57514 bdc2c6b40bf2
parent 57492 74bf65a1910a
child 61076 bdc1e2f0a86a
--- a/src/HOL/Quotient_Examples/Quotient_Int.thy	Sat Jul 05 10:09:01 2014 +0200
+++ b/src/HOL/Quotient_Examples/Quotient_Int.thy	Sat Jul 05 11:01:53 2014 +0200
@@ -60,7 +60,7 @@
   apply(hypsubst_thin)
   apply(rename_tac u v w x y z)
   apply(subgoal_tac "u*w + z*w = y*w + v*w  &  u*x + z*x = y*x + v*x")
-  apply(simp add: mult_ac)
+  apply(simp add: ac_simps)
   apply(simp add: add_mult_distrib [symmetric])
 done
 
@@ -73,7 +73,7 @@
   apply(hypsubst_thin)
   apply(rename_tac u v w x y z)
   apply(subgoal_tac "u*w + z*w = y*w + v*w  &  u*x + z*x = y*x + v*x")
-  apply(simp add: mult_ac)
+  apply(simp add: ac_simps)
   apply(simp add: add_mult_distrib [symmetric])
 done