src/HOL/UNITY/Union.thy
changeset 35434 a4babce15c67
parent 35427 ad039d29e01c
child 36866 426d5781bb25
--- a/src/HOL/UNITY/Union.thy	Wed Mar 03 00:50:47 2010 +0100
+++ b/src/HOL/UNITY/Union.thy	Wed Mar 03 12:02:59 2010 +0100
@@ -35,7 +35,7 @@
   safety_prop :: "'a program set => bool"
     "safety_prop X == SKIP: X & (\<forall>G. Acts G \<subseteq> UNION X Acts --> G \<in> X)"
 
-notation
+notation (xsymbols)
   SKIP  ("\<bottom>") and
   Join  (infixl "\<squnion>" 65)