src/HOL/Lattice/Orders.thy
changeset 21210 c17fd2df4e9e
parent 20523 36a59e5d0039
child 35317 d57da4abb47d
--- a/src/HOL/Lattice/Orders.thy	Tue Nov 07 11:47:56 2006 +0100
+++ b/src/HOL/Lattice/Orders.thy	Tue Nov 07 11:47:57 2006 +0100
@@ -21,7 +21,7 @@
 axclass leq < type
 consts
   leq :: "'a::leq \<Rightarrow> 'a \<Rightarrow> bool"  (infixl "[=" 50)
-const_syntax (xsymbols)
+notation (xsymbols)
   leq  (infixl "\<sqsubseteq>" 50)
 
 axclass quasi_order < leq