src/HOL/HOL.thy
changeset 21404 eb85850d3eb7
parent 21250 a268f6288fb6
child 21410 c212b002fc8c
--- a/src/HOL/HOL.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/HOL.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -58,27 +58,27 @@
   "op ="  (infix "=" 50)
 
 abbreviation
-  not_equal     :: "['a, 'a] => bool"               (infixl "~=" 50)
+  not_equal :: "['a, 'a] => bool"  (infixl "~=" 50) where
   "x ~= y == ~ (x = y)"
 
 notation (output)
   not_equal  (infix "~=" 50)
 
 notation (xsymbols)
-  Not  ("\<not> _" [40] 40)
-  "op &"  (infixr "\<and>" 35)
-  "op |"  (infixr "\<or>" 30)
-  "op -->"  (infixr "\<longrightarrow>" 25)
+  Not  ("\<not> _" [40] 40) and
+  "op &"  (infixr "\<and>" 35) and
+  "op |"  (infixr "\<or>" 30) and
+  "op -->"  (infixr "\<longrightarrow>" 25) and
   not_equal  (infix "\<noteq>" 50)
 
 notation (HTML output)
-  Not  ("\<not> _" [40] 40)
-  "op &"  (infixr "\<and>" 35)
-  "op |"  (infixr "\<or>" 30)
+  Not  ("\<not> _" [40] 40) and
+  "op &"  (infixr "\<and>" 35) and
+  "op |"  (infixr "\<or>" 30) and
   not_equal  (infix "\<noteq>" 50)
 
 abbreviation (iff)
-  iff :: "[bool, bool] => bool"  (infixr "<->" 25)
+  iff :: "[bool, bool] => bool"  (infixr "<->" 25) where
   "A <-> B == A = B"
 
 notation (xsymbols)