src/FOL/IFOL.thy
changeset 21404 eb85850d3eb7
parent 21210 c17fd2df4e9e
child 21524 7843e2fd14a9
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
    43   Ex            :: "('a => o) => o"             (binder "EX " 10)
    43   Ex            :: "('a => o) => o"             (binder "EX " 10)
    44   Ex1           :: "('a => o) => o"             (binder "EX! " 10)
    44   Ex1           :: "('a => o) => o"             (binder "EX! " 10)
    45 
    45 
    46 
    46 
    47 abbreviation
    47 abbreviation
    48   not_equal     :: "['a, 'a] => o"              (infixl "~=" 50)
    48   not_equal :: "['a, 'a] => o"  (infixl "~=" 50) where
    49   "x ~= y == ~ (x = y)"
    49   "x ~= y == ~ (x = y)"
    50 
    50 
    51 notation (xsymbols)
    51 notation (xsymbols)
    52   not_equal  (infixl "\<noteq>" 50)
    52   not_equal  (infixl "\<noteq>" 50)
    53 
    53