src/HOL/String.thy
changeset 37743 0a3fa8fbcdc5
parent 36176 3fe7e97ccca8
child 38808 89ae86205739
child 38857 97775f3e8722
--- a/src/HOL/String.thy	Thu Jul 08 16:17:44 2010 +0200
+++ b/src/HOL/String.thy	Thu Jul 08 16:19:23 2010 +0200
@@ -219,4 +219,16 @@
 
 hide_type (open) literal
 
+
+text {* Code generator setup *}
+
+code_modulename SML
+  String String
+
+code_modulename OCaml
+  String String
+
+code_modulename Haskell
+  String String
+
 end
\ No newline at end of file