src/HOL/Library/EfficientNat.thy
changeset 23711 dc452e8641aa
parent 23591 d32a85385e17
child 23809 6104514a1f5f
--- a/src/HOL/Library/EfficientNat.thy	Tue Jul 10 17:30:51 2007 +0200
+++ b/src/HOL/Library/EfficientNat.thy	Tue Jul 10 17:30:52 2007 +0200
@@ -385,14 +385,17 @@
 *}
 (*>*)
 
+
 subsection {* Module names *}
 
 code_modulename SML
   Nat Integer
+  Divides Integer
   EfficientNat Integer
 
 code_modulename OCaml
   Nat Integer
+  Divides Integer
   EfficientNat Integer
 
 code_modulename Haskell