src/HOL/Divides.thy
changeset 35050 9f841f20dca6
parent 34982 7b8c366e34a2
child 35216 7641e8d831d2
--- a/src/HOL/Divides.thy	Mon Feb 08 17:12:32 2010 +0100
+++ b/src/HOL/Divides.thy	Mon Feb 08 17:12:38 2010 +0100
@@ -657,7 +657,7 @@
   val trans = trans;
 
   val prove_eq_sums = Arith_Data.prove_conv2 all_tac (Arith_Data.simp_all_tac
-    (@{thm monoid_add_class.add_0_left} :: @{thm monoid_add_class.add_0_right} :: @{thms add_ac}))
+    (@{thm add_0_left} :: @{thm add_0_right} :: @{thms add_ac}))
 
 end)
 
@@ -1655,8 +1655,8 @@
 lemmas arithmetic_simps =
   arith_simps
   add_special
-  OrderedGroup.add_0_left
-  OrderedGroup.add_0_right
+  add_0_left
+  add_0_right
   mult_zero_left
   mult_zero_right
   mult_1_left