src/HOL/Library/ML_String.thy
changeset 24219 e558fe311376
parent 23854 688a8a7bcd4e
child 24717 56ba87ec8d31
--- a/src/HOL/Library/ML_String.thy	Fri Aug 10 17:04:24 2007 +0200
+++ b/src/HOL/Library/ML_String.thy	Fri Aug 10 17:04:34 2007 +0200
@@ -60,7 +60,7 @@
     @{const_name NibbleC}, @{const_name NibbleD},
     @{const_name NibbleE}, @{const_name NibbleF}];
 in
-  CodegenSerializer.add_pretty_ml_string "SML"
+  CodeTarget.add_pretty_ml_string "SML"
     charr nibbles @{const_name Nil} @{const_name Cons} @{const_name STR}
 end
 *}