src/HOL/Int.thy
changeset 70354 9497a6334a26
parent 69791 195aeee8b30a
child 70356 4a327c061870
equal deleted inserted replaced
70353:7aa64296b9b0 70354:9497a6334a26
  1084 end
  1084 end
  1085 
  1085 
  1086 
  1086 
  1087 subsection \<open>Setting up simplification procedures\<close>
  1087 subsection \<open>Setting up simplification procedures\<close>
  1088 
  1088 
  1089 lemmas of_int_simps =
  1089 lemmas of_int_simps [no_atp] =
  1090   of_int_0 of_int_1 of_int_add of_int_mult
  1090   of_int_0 of_int_1 of_int_add of_int_mult
  1091 
  1091 
  1092 ML_file \<open>Tools/int_arith.ML\<close>
  1092 ML_file \<open>Tools/int_arith.ML\<close>
  1093 declaration \<open>K Int_Arith.setup\<close>
  1093 declaration \<open>K Int_Arith.setup\<close>
  1094 
  1094