src/HOL/Set.thy
changeset 25360 b8251517f508
parent 25287 094dab519ff5
child 25460 b80087af2274
--- a/src/HOL/Set.thy	Thu Nov 08 22:57:45 2007 +0100
+++ b/src/HOL/Set.thy	Fri Nov 09 13:41:27 2007 +0100
@@ -2255,6 +2255,7 @@
   "Union A = UNION A (\<lambda>x. x)"
   by auto
 
+code_reserved SML union inter (* Avoid clashes with ML infixes *)
 
 subsection {* Basic ML bindings *}