src/HOL/Library/Word.thy
changeset 21210 c17fd2df4e9e
parent 20485 3078fd2eec7b
child 21404 eb85850d3eb7
--- a/src/HOL/Library/Word.thy	Tue Nov 07 11:47:56 2006 +0100
+++ b/src/HOL/Library/Word.thy	Tue Nov 07 11:47:57 2006 +0100
@@ -56,13 +56,13 @@
   bitor  :: "bit => bit => bit" (infixr "bitor"  30)
   bitxor :: "bit => bit => bit" (infixr "bitxor" 30)
 
-const_syntax (xsymbols)
+notation (xsymbols)
   bitnot ("\<not>\<^sub>b _" [40] 40)
   bitand (infixr "\<and>\<^sub>b" 35)
   bitor  (infixr "\<or>\<^sub>b" 30)
   bitxor (infixr "\<oplus>\<^sub>b" 30)
 
-const_syntax (HTML output)
+notation (HTML output)
   bitnot ("\<not>\<^sub>b _" [40] 40)
   bitand (infixr "\<and>\<^sub>b" 35)
   bitor  (infixr "\<or>\<^sub>b" 30)