src/HOL/ex/Numeral.thy
changeset 33523 96730ad673be
parent 33346 c5cd93763e71
child 35028 108662d50512
--- a/src/HOL/ex/Numeral.thy	Sun Nov 08 18:43:42 2009 +0100
+++ b/src/HOL/ex/Numeral.thy	Sun Nov 08 19:15:37 2009 +0100
@@ -923,22 +923,21 @@
 
 declare Suc_of_num [simp]
 
-thm numeral
-
 
 subsection {* Simplification Procedures *}
 
 subsubsection {* Reorientation of equalities *}
 
 setup {*
-  ReorientProc.add
+  Reorient_Proc.add
     (fn Const(@{const_name of_num}, _) $ _ => true
       | Const(@{const_name uminus}, _) $
           (Const(@{const_name of_num}, _) $ _) => true
       | _ => false)
 *}
 
-simproc_setup reorient_num ("of_num n = x" | "- of_num m = y") = ReorientProc.proc
+simproc_setup reorient_num ("of_num n = x" | "- of_num m = y") = Reorient_Proc.proc
+
 
 subsubsection {* Constant folding for multiplication in semirings *}