src/HOL/Lattice/Lattice.thy
changeset 12114 a8e860c86252
parent 11441 54b236801671
child 12338 de0f4a63baa5
--- a/src/HOL/Lattice/Lattice.thy	Fri Nov 09 00:06:15 2001 +0100
+++ b/src/HOL/Lattice/Lattice.thy	Fri Nov 09 00:09:47 2001 +0100
@@ -27,7 +27,7 @@
 consts
   meet :: "'a::lattice \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "&&" 70)
   join :: "'a::lattice \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "||" 65)
-syntax (symbols)
+syntax (xsymbols)
   meet :: "'a::lattice \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "\<sqinter>" 70)
   join :: "'a::lattice \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "\<squnion>" 65)
 defs