| changeset 31024 | 0fdf666e08bf |
| parent 31021 | 53642251a04f |
| child 31065 | d87465cbfc9e |
--- a/src/HOL/Int.thy Wed Apr 29 13:36:29 2009 -0700 +++ b/src/HOL/Int.thy Wed Apr 29 17:15:01 2009 -0700 @@ -1518,6 +1518,13 @@ use "Tools/int_arith.ML" declaration {* K Int_Arith.setup *} +setup {* + ReorientProc.add + (fn Const(@{const_name number_of}, _) $ _ => true | _ => false) +*} + +simproc_setup reorient_numeral ("number_of w = x") = ReorientProc.proc + subsection{*Lemmas About Small Numerals*}