src/HOL/Library/ExecutableSet.thy
changeset 19137 f92919b141b2
parent 19041 1a8f08f9f8af
child 19233 77ca20b0ed77
--- a/src/HOL/Library/ExecutableSet.thy	Sat Feb 25 15:19:00 2006 +0100
+++ b/src/HOL/Library/ExecutableSet.thy	Sat Feb 25 15:19:19 2006 +0100
@@ -82,7 +82,7 @@
   "inter [] ys = []"
   "inter (x#xs) ys = (let xs' = inter xs ys in if member ys x then x#xs' else xs')"
 
-code_syntax_const "insert"
+code_syntax_const insert
   ml ("{*insert_*}")
   haskell ("{*insert_*}")
 
@@ -90,7 +90,7 @@
   ml ("{*foldr insert_*}")
   haskell ("{*foldr insert_*}")
 
-code_syntax_const "op -" :: "'a set \<Rightarrow> 'a set \<Rightarrow> 'a set"
+code_syntax_const "op - :: 'a set \<Rightarrow> 'a set \<Rightarrow> 'a set"
   ml ("{*(flip o foldr) remove*}")
   haskell ("{*(flip o foldr) remove*}")
 
@@ -98,19 +98,19 @@
   ml ("{*inter*}")
   haskell ("{*inter*}")
 
-code_syntax_const "image"
+code_syntax_const image
   ml ("{*\<lambda>f. foldr (insert_ o f)*}")
   haskell ("{*\<lambda>f. foldr (insert_ o f)*}")
 
-code_syntax_const "INTER"
+code_syntax_const INTER
   ml ("{*\<lambda>xs f.  foldr (inter o f) xs*}")
   haskell ("{*\<lambda>xs f.  foldr (inter o f) xs*}")
 
-code_syntax_const "UNION"
+code_syntax_const UNION
   ml ("{*\<lambda>xs f.  foldr (foldr insert_ o f) xs*}")
   haskell ("{*\<lambda>xs f.  foldr (foldr insert_ o f) xs*}")
 
-code_primconst "Ball"
+code_primconst Ball
 ml {*
 fun `_` [] f = true
   | `_` (x::xs) f = f x andalso `_` xs f;
@@ -119,7 +119,7 @@
 `_` = flip all
 *}
 
-code_primconst "Bex"
+code_primconst Bex
 ml {*
 fun `_` [] f = false
   | `_` (x::xs) f = f x orelse `_` xs f;