src/HOL/Num.thy
changeset 78099 4d9349989d94
parent 75669 43f5dfb7fa35
child 79590 b14c4cb37d99
--- a/src/HOL/Num.thy	Tue May 23 20:11:15 2023 +0200
+++ b/src/HOL/Num.thy	Tue May 23 21:43:36 2023 +0200
@@ -1394,7 +1394,7 @@
 \<close>
 
 simproc_setup reorient_numeral ("numeral w = x" | "- numeral w = y") =
-  Reorient_Proc.proc
+  \<open>K Reorient_Proc.proc\<close>
 
 
 subsubsection \<open>Simplification of arithmetic operations on integer constants\<close>