src/HOL/OrderedGroup.thy
changeset 33364 2bd12592c5e8
parent 32642 026e7c6a6d08
child 34146 14595e0c27e8
--- a/src/HOL/OrderedGroup.thy	Fri Oct 30 14:02:42 2009 +0100
+++ b/src/HOL/OrderedGroup.thy	Fri Oct 30 18:32:40 2009 +0100
@@ -1409,4 +1409,13 @@
   Addsimprocs [ab_group_add_cancel.sum_conv, ab_group_add_cancel.rel_conv];
 *}
 
+code_modulename SML
+  OrderedGroup Arith
+
+code_modulename OCaml
+  OrderedGroup Arith
+
+code_modulename Haskell
+  OrderedGroup Arith
+
 end