src/HOL/Num.thy
changeset 59621 291934bac95e
parent 58889 5b7a9633cfa8
child 59867 58043346ca64
equal deleted inserted replaced
59620:92d7d8e4f1bf 59621:291934bac95e
  1196 declaration {*
  1196 declaration {*
  1197 let 
  1197 let 
  1198   fun number_of thy T n =
  1198   fun number_of thy T n =
  1199     if not (Sign.of_sort thy (T, @{sort numeral}))
  1199     if not (Sign.of_sort thy (T, @{sort numeral}))
  1200     then raise CTERM ("number_of", [])
  1200     then raise CTERM ("number_of", [])
  1201     else Numeral.mk_cnumber (Thm.ctyp_of thy T) n;
  1201     else Numeral.mk_cnumber (Thm.global_ctyp_of thy T) n;
  1202 in
  1202 in
  1203   K (
  1203   K (
  1204     Lin_Arith.add_simps (@{thms arith_simps} @ @{thms more_arith_simps}
  1204     Lin_Arith.add_simps (@{thms arith_simps} @ @{thms more_arith_simps}
  1205       @ @{thms rel_simps}
  1205       @ @{thms rel_simps}
  1206       @ @{thms pred_numeral_simps}
  1206       @ @{thms pred_numeral_simps}