adapted to multiple results;
authorwenzelm
Sun, 11 Nov 2001 21:37:44 +0100
changeset 12148 a57873aec3bf
parent 12147 64e69a8a945f
child 12149 7cf8574102d5
adapted to multiple results;
src/Pure/Isar/skip_proof.ML
--- a/src/Pure/Isar/skip_proof.ML	Sun Nov 11 21:37:20 2001 +0100
+++ b/src/Pure/Isar/skip_proof.ML	Sun Nov 11 21:37:44 2001 +0100
@@ -12,9 +12,9 @@
   val make_thm: theory -> term -> thm
   val cheat_tac: theory -> tactic
   val prove: theory -> string list -> term list -> term -> (thm list -> tactic) -> thm
-  val local_skip_proof: (Proof.context -> {kind: string, name: string, thm: thm} -> unit) *
+  val local_skip_proof: (Proof.context -> string * (string * thm list) list -> unit) *
     (Proof.context -> thm -> unit) -> Proof.state -> Proof.state Seq.seq
-  val global_skip_proof: Proof.state -> theory * {kind: string, name: string, thm: thm}
+  val global_skip_proof: Proof.state -> theory * (string * (string * thm list) list)
   val setup: (theory -> theory) list
 end;