src/HOL/Product_Type.thy
changeset 18757 f0d901bc0686
parent 18708 4b3dadb4fe33
child 18963 3adfc9dfb30a
--- a/src/HOL/Product_Type.thy	Mon Jan 23 14:06:40 2006 +0100
+++ b/src/HOL/Product_Type.thy	Mon Jan 23 14:07:52 2006 +0100
@@ -798,13 +798,13 @@
 code_syntax_tyco
   *
     ml (infix 2 "*")
-    haskell (atom "(__,/ __)")
+    haskell (target_atom "(__,/ __)")
 
 code_syntax_const
   fst
-    haskell (atom "fst")
+    haskell (target_atom "fst")
   snd
-    haskell (atom "snd")
+    haskell (target_atom "snd")
 
 ML {*