src/HOL/List.thy
changeset 78800 0b3700d31758
parent 78099 4d9349989d94
child 78801 42ae6e0ecfd4
--- a/src/HOL/List.thy	Thu Oct 19 16:31:17 2023 +0200
+++ b/src/HOL/List.thy	Thu Oct 19 17:06:39 2023 +0200
@@ -557,7 +557,7 @@
 
 signature LIST_TO_SET_COMPREHENSION =
 sig
-  val simproc : Proof.context -> cterm -> thm option
+  val simproc : Simplifier.proc
 end
 
 structure List_to_Set_Comprehension : LIST_TO_SET_COMPREHENSION =