src/Provers/Arith/fast_lin_arith.ML
changeset 78800 0b3700d31758
parent 78133 0a098088745b
--- a/src/Provers/Arith/fast_lin_arith.ML	Thu Oct 19 16:31:17 2023 +0200
+++ b/src/Provers/Arith/fast_lin_arith.ML	Thu Oct 19 17:06:39 2023 +0200
@@ -93,7 +93,7 @@
 sig
   val prems_lin_arith_tac: Proof.context -> int -> tactic
   val lin_arith_tac: Proof.context -> int -> tactic
-  val lin_arith_simproc: Proof.context -> cterm -> thm option
+  val lin_arith_simproc: Simplifier.proc
   val map_data:
     ({add_mono_thms: thm list, mult_mono_thms: thm list, inj_thms: thm list,
       lessD: thm list, neqE: thm list, simpset: simpset,