src/HOL/Library/ExecutableSet.thy
changeset 18757 f0d901bc0686
parent 18702 7dc7dcd63224
child 18772 f0dd51087eb3
--- a/src/HOL/Library/ExecutableSet.thy	Mon Jan 23 14:06:40 2006 +0100
+++ b/src/HOL/Library/ExecutableSet.thy	Mon Jan 23 14:07:52 2006 +0100
@@ -29,11 +29,11 @@
 
 code_syntax_tyco set
   ml ("_ list")
-  haskell (atom "[_]")
+  haskell (target_atom "[_]")
 
 code_syntax_const "{}"
-  ml (atom "[]")
-  haskell (atom "[]")
+  ml (target_atom "[]")
+  haskell (target_atom "[]")
 
 consts_code
   "{}"      ("[]")