local qed; print rule;
authorwenzelm
Mon, 12 Jul 1999 22:28:56 +0200
changeset 6984 26d43e26ea61
parent 6983 7f28cd9cfe72
child 6985 2af6405a6ef3
local qed; print rule;
src/Pure/Isar/skip_proof.ML
--- a/src/Pure/Isar/skip_proof.ML	Mon Jul 12 22:28:38 1999 +0200
+++ b/src/Pure/Isar/skip_proof.ML	Mon Jul 12 22:28:56 1999 +0200
@@ -7,7 +7,7 @@
 
 signature SKIP_PROOF =
 sig
-  val local_skip_proof: ({kind: string, name: string, thm: thm} -> unit)
+  val local_skip_proof: ({kind: string, name: string, thm: thm} -> unit) * (thm -> unit)
     -> Proof.state -> Proof.state Seq.seq
   val global_skip_proof: Proof.state -> theory * {kind: string, name: string, thm: thm}
   val setup: (theory -> theory) list