src/HOL/Library/Lattice_Syntax.thy
changeset 61955 e96292f32c3c
parent 60500 903bb1495239
child 66453 cc19f7ca2ed6
--- a/src/HOL/Library/Lattice_Syntax.thy	Mon Dec 28 19:23:15 2015 +0100
+++ b/src/HOL/Library/Lattice_Syntax.thy	Mon Dec 28 21:47:32 2015 +0100
@@ -14,7 +14,7 @@
   Inf  ("\<Sqinter>_" [900] 900) and
   Sup  ("\<Squnion>_" [900] 900)
 
-syntax (xsymbols)
+syntax
   "_INF1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3\<Sqinter>_./ _)" [0, 10] 10)
   "_INF"      :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b"  ("(3\<Sqinter>_\<in>_./ _)" [0, 0, 10] 10)
   "_SUP1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3\<Squnion>_./ _)" [0, 10] 10)