src/HOL/Int.thy
changeset 29039 8b9207f82a78
parent 28988 13d6f120992b
child 29040 286c669d3a7a
equal deleted inserted replaced
29038:90f42c138585 29039:8b9207f82a78
  1252   also have "... = (w < 0)" by (simp only: of_int_less_iff odd_less_0)
  1252   also have "... = (w < 0)" by (simp only: of_int_less_iff odd_less_0)
  1253   finally show ?thesis
  1253   finally show ?thesis
  1254   by (simp add: neg_def number_of_eq numeral_simps)
  1254   by (simp add: neg_def number_of_eq numeral_simps)
  1255 qed
  1255 qed
  1256 
  1256 
  1257 lemmas neg_simps =
  1257 lemmas neg_simps [simp] =
  1258   not_neg_0 not_neg_1
  1258   not_neg_0 not_neg_1
  1259   not_neg_number_of_Pls neg_number_of_Min
  1259   not_neg_number_of_Pls neg_number_of_Min
  1260   neg_number_of_Bit0 neg_number_of_Bit1
  1260   neg_number_of_Bit0 neg_number_of_Bit1
  1261 
  1261 
  1262 text {* Less-Than or Equals *}
  1262 text {* Less-Than or Equals *}
  1323 
  1323 
  1324 lemmas rel_simps [simp] = 
  1324 lemmas rel_simps [simp] = 
  1325   less_number_of less_bin_simps
  1325   less_number_of less_bin_simps
  1326   le_number_of le_bin_simps
  1326   le_number_of le_bin_simps
  1327   eq_number_of_eq eq_bin_simps
  1327   eq_number_of_eq eq_bin_simps
  1328   iszero_simps neg_simps
  1328   iszero_simps
  1329 
  1329 
  1330 
  1330 
  1331 subsubsection {* Simplification of arithmetic when nested to the right. *}
  1331 subsubsection {* Simplification of arithmetic when nested to the right. *}
  1332 
  1332 
  1333 lemma add_number_of_left [simp]:
  1333 lemma add_number_of_left [simp]: