src/HOL/List.thy
changeset 28064 d4a6460c53d1
parent 28054 2b84d34c5d02
child 28068 f6b2d1995171
--- a/src/HOL/List.thy	Fri Aug 29 20:36:08 2008 +0200
+++ b/src/HOL/List.thy	Mon Sep 01 10:18:37 2008 +0200
@@ -3450,7 +3450,7 @@
   (Haskell "[]")
 
 setup {*
-  fold (fn target => Code_Target.add_pretty_list target
+  fold (fn target => Code_Target.add_literal_list target
     @{const_name Nil} @{const_name Cons}
   ) ["SML", "OCaml", "Haskell"]
 *}