src/HOL/Library/Word.thy
changeset 25162 ad4d5365d9d8
parent 25134 3d4953e88449
child 25595 6c48275f9c76
equal deleted inserted replaced
25161:aa8474398030 25162:ad4d5365d9d8
   477       proof (simp_all)
   477       proof (simp_all)
   478         assume "n mod 2 = 0"
   478         assume "n mod 2 = 0"
   479         with mod_div_equality [of n 2]
   479         with mod_div_equality [of n 2]
   480         show "n div 2 * 2 = n" by simp
   480         show "n div 2 * 2 = n" by simp
   481       next
   481       next
   482         assume "n mod 2 \<noteq> 0"
   482         assume "n mod 2 = Suc 0"
   483         with mod_div_equality [of n 2]
   483         with mod_div_equality [of n 2]
   484         show "Suc (n div 2 * 2) = n" by arith
   484         show "Suc (n div 2 * 2) = n" by arith
   485       qed
   485       qed
   486   qed
   486   qed
   487 qed
   487 qed