src/HOL/Int.thy
changeset 69605 a96320074298
parent 69593 3dda49e08b9d
child 69700 7a92cbec7030
equal deleted inserted replaced
69604:d80b2df54d31 69605:a96320074298
  1079 subsection \<open>Setting up simplification procedures\<close>
  1079 subsection \<open>Setting up simplification procedures\<close>
  1080 
  1080 
  1081 lemmas of_int_simps =
  1081 lemmas of_int_simps =
  1082   of_int_0 of_int_1 of_int_add of_int_mult
  1082   of_int_0 of_int_1 of_int_add of_int_mult
  1083 
  1083 
  1084 ML_file "Tools/int_arith.ML"
  1084 ML_file \<open>Tools/int_arith.ML\<close>
  1085 declaration \<open>K Int_Arith.setup\<close>
  1085 declaration \<open>K Int_Arith.setup\<close>
  1086 
  1086 
  1087 simproc_setup fast_arith
  1087 simproc_setup fast_arith
  1088   ("(m::'a::linordered_idom) < n" |
  1088   ("(m::'a::linordered_idom) < n" |
  1089     "(m::'a::linordered_idom) \<le> n" |
  1089     "(m::'a::linordered_idom) \<le> n" |