diff -r dd58f13a8eb4 -r eb85850d3eb7 src/HOL/HOL.thy --- 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 ("\ _" [40] 40) - "op &" (infixr "\" 35) - "op |" (infixr "\" 30) - "op -->" (infixr "\" 25) + Not ("\ _" [40] 40) and + "op &" (infixr "\" 35) and + "op |" (infixr "\" 30) and + "op -->" (infixr "\" 25) and not_equal (infix "\" 50) notation (HTML output) - Not ("\ _" [40] 40) - "op &" (infixr "\" 35) - "op |" (infixr "\" 30) + Not ("\ _" [40] 40) and + "op &" (infixr "\" 35) and + "op |" (infixr "\" 30) and not_equal (infix "\" 50) abbreviation (iff) - iff :: "[bool, bool] => bool" (infixr "<->" 25) + iff :: "[bool, bool] => bool" (infixr "<->" 25) where "A <-> B == A = B" notation (xsymbols)