src/HOL/Library/Parity.thy
changeset 21404 eb85850d3eb7
parent 21263 de65ce2bfb32
child 22390 378f34b1e380
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
    20 defs (overloaded)
    20 defs (overloaded)
    21   even_def: "even (x::int) == x mod 2 = 0"
    21   even_def: "even (x::int) == x mod 2 = 0"
    22   even_nat_def: "even (x::nat) == even (int x)"
    22   even_nat_def: "even (x::nat) == even (int x)"
    23 
    23 
    24 abbreviation
    24 abbreviation
    25   odd :: "'a::even_odd => bool"
    25   odd :: "'a::even_odd => bool" where
    26   "odd x == \<not> even x"
    26   "odd x == \<not> even x"
    27 
    27 
    28 
    28 
    29 subsection {* Even and odd are mutually exclusive *}
    29 subsection {* Even and odd are mutually exclusive *}
    30 
    30