src/HOL/Int.thy
changeset 33523 96730ad673be
parent 33364 2bd12592c5e8
child 33657 a4179bf442d1
--- a/src/HOL/Int.thy	Sun Nov 08 18:43:42 2009 +0100
+++ b/src/HOL/Int.thy	Sun Nov 08 19:15:37 2009 +0100
@@ -1502,11 +1502,11 @@
 declaration {* K Int_Arith.setup *}
 
 setup {*
-  ReorientProc.add
+  Reorient_Proc.add
     (fn Const (@{const_name number_of}, _) $ _ => true | _ => false)
 *}
 
-simproc_setup reorient_numeral ("number_of w = x") = ReorientProc.proc
+simproc_setup reorient_numeral ("number_of w = x") = Reorient_Proc.proc
 
 
 subsection{*Lemmas About Small Numerals*}