src/HOL/Num.thy
changeset 64238 b60a9752b6d0
parent 64178 12e6c3bbb488
child 66283 adf3155c57e2
equal deleted inserted replaced
64237:c1b5165b73db 64238:b60a9752b6d0
  1215     else Numeral.mk_cnumber (Thm.ctyp_of ctxt T) n;
  1215     else Numeral.mk_cnumber (Thm.ctyp_of ctxt T) n;
  1216 in
  1216 in
  1217   K (
  1217   K (
  1218     Lin_Arith.add_simps
  1218     Lin_Arith.add_simps
  1219       @{thms arith_simps more_arith_simps rel_simps pred_numeral_simps
  1219       @{thms arith_simps more_arith_simps rel_simps pred_numeral_simps
  1220         arith_special numeral_One of_nat_simps}
  1220         arith_special numeral_One of_nat_simps uminus_numeral_One}
  1221     #> Lin_Arith.add_simps
  1221     #> Lin_Arith.add_simps
  1222       @{thms Suc_numeral Let_numeral Let_neg_numeral Let_0 Let_1
  1222       @{thms Suc_numeral Let_numeral Let_neg_numeral Let_0 Let_1
  1223         le_Suc_numeral le_numeral_Suc less_Suc_numeral less_numeral_Suc
  1223         le_Suc_numeral le_numeral_Suc less_Suc_numeral less_numeral_Suc
  1224         Suc_eq_numeral eq_numeral_Suc mult_Suc mult_Suc_right of_nat_numeral}
  1224         Suc_eq_numeral eq_numeral_Suc mult_Suc mult_Suc_right of_nat_numeral}
  1225     #> Lin_Arith.set_number_of number_of)
  1225     #> Lin_Arith.set_number_of number_of)