src/HOL/Word/Word.thy
changeset 46647 de514a98f6b6
parent 46646 0abbf6dd09ee
child 46648 689ebcbd6343
equal deleted inserted replaced
46646:0abbf6dd09ee 46647:de514a98f6b6
  1197 lemmas uint_div_alt = word_div_def [THEN trans [OF uint_cong int_word_uint]]
  1197 lemmas uint_div_alt = word_div_def [THEN trans [OF uint_cong int_word_uint]]
  1198 lemmas uint_mod_alt = word_mod_def [THEN trans [OF uint_cong int_word_uint]]
  1198 lemmas uint_mod_alt = word_mod_def [THEN trans [OF uint_cong int_word_uint]]
  1199 
  1199 
  1200 lemma word_pred_0_n1: "word_pred 0 = word_of_int -1"
  1200 lemma word_pred_0_n1: "word_pred 0 = word_of_int -1"
  1201   unfolding word_pred_def uint_eq_0 pred_def by simp
  1201   unfolding word_pred_def uint_eq_0 pred_def by simp
  1202 
       
  1203 lemma word_pred_0_Min: "word_pred 0 = word_of_int Int.Min"
       
  1204   by (simp add: word_pred_0_n1 number_of_eq)
       
  1205 
       
  1206 lemma word_m1_Min: "- 1 = word_of_int Int.Min"
       
  1207   unfolding Min_def by (simp only: word_of_int_hom_syms)
       
  1208 
  1202 
  1209 lemma succ_pred_no [simp]:
  1203 lemma succ_pred_no [simp]:
  1210   "word_succ (number_of bin) = number_of (Int.succ bin) & 
  1204   "word_succ (number_of bin) = number_of (Int.succ bin) & 
  1211     word_pred (number_of bin) = number_of (Int.pred bin)"
  1205     word_pred (number_of bin) = number_of (Int.pred bin)"
  1212   unfolding word_number_of_def Int.succ_def Int.pred_def
  1206   unfolding word_number_of_def Int.succ_def Int.pred_def