src/HOL/Divides.thy
changeset 52435 6646bb548c6b
parent 52398 656e5e171f19
child 53066 1f61a923c2d6
--- a/src/HOL/Divides.thy	Sun Jun 23 21:16:06 2013 +0200
+++ b/src/HOL/Divides.thy	Sun Jun 23 21:16:07 2013 +0200
@@ -2381,13 +2381,8 @@
   then show ?thesis by (simp add: divmod_int_pdivmod)
 qed
 
-code_modulename SML
-  Divides Arith
-
-code_modulename OCaml
-  Divides Arith
-
-code_modulename Haskell
-  Divides Arith
+code_identifier
+  code_module Divides \<rightharpoonup> (SML) Arith and (OCaml) Arith and (Haskell) Arith
 
 end
+