unused (see d12c58e12c51);
authorwenzelm
Tue, 13 Aug 2024 15:50:25 +0200
changeset 80698 2d2f476ab56e
parent 80697 48eaf5c85d6e
child 80699 34db40261287
unused (see d12c58e12c51);
src/Pure/raw_simplifier.ML
--- a/src/Pure/raw_simplifier.ML	Tue Aug 13 15:42:55 2024 +0200
+++ b/src/Pure/raw_simplifier.ML	Tue Aug 13 15:50:25 2024 +0200
@@ -20,7 +20,6 @@
   val mk_rrules: Proof.context -> thm list -> rrule list
   val eq_rrule: rrule * rrule -> bool
   type proc = Proof.context -> cterm -> thm option
-  type procedure
   type solver
   val mk_solver: string -> (Proof.context -> int -> tactic) -> solver
   type simpset