src/HOL/Library/ExecutableSet.thy
changeset 21008 330a8a6dd53c
parent 20934 2b872c161747
child 21046 fe1db2f991a7
--- a/src/HOL/Library/ExecutableSet.thy	Thu Oct 12 22:57:45 2006 +0200
+++ b/src/HOL/Library/ExecutableSet.thy	Fri Oct 13 09:02:21 2006 +0200
@@ -230,6 +230,11 @@
 
 section {* code generator setup *}
 
+ML {*
+nonfix inter;
+nonfix union;
+*}
+
 code_constname
   "ExecutableSet.member" "List.member"
   "ExecutableSet.insertl" "List.insertl"