src/HOL/List.thy
changeset 28054 2b84d34c5d02
parent 27715 087db5aacac3
child 28064 d4a6460c53d1
--- a/src/HOL/List.thy	Thu Aug 28 22:08:11 2008 +0200
+++ b/src/HOL/List.thy	Thu Aug 28 22:09:20 2008 +0200
@@ -3450,7 +3450,7 @@
   (Haskell "[]")
 
 setup {*
-  fold (fn target => CodeTarget.add_pretty_list target
+  fold (fn target => Code_Target.add_pretty_list target
     @{const_name Nil} @{const_name Cons}
   ) ["SML", "OCaml", "Haskell"]
 *}