src/HOL/Library/Pretty_Int.thy
changeset 24219 e558fe311376
parent 23859 fc44fa554ca8
child 24423 ae9cd0e92423
--- a/src/HOL/Library/Pretty_Int.thy	Fri Aug 10 17:04:24 2007 +0200
+++ b/src/HOL/Library/Pretty_Int.thy	Fri Aug 10 17:04:34 2007 +0200
@@ -24,7 +24,7 @@
   (Haskell -)
 
 setup {*
-  fold (fn target => CodegenSerializer.add_pretty_numeral target true
+  fold (fn target => CodeTarget.add_pretty_numeral target true
     (@{const_name number_of}, @{typ "int \<Rightarrow> int"})
     @{const_name Numeral.B0} @{const_name Numeral.B1}
     @{const_name Numeral.Pls} @{const_name Numeral.Min}