src/Doc/Implementation/Tactic.thy
changeset 59780 23b67731f4f0
parent 59763 56d2c357e6b5
child 59902 6afbe5a99139
--- a/src/Doc/Implementation/Tactic.thy	Mon Mar 23 10:16:20 2015 +0100
+++ b/src/Doc/Implementation/Tactic.thy	Mon Mar 23 13:30:59 2015 +0100
@@ -395,15 +395,21 @@
 text %mlref \<open>
   \begin{mldecls}
   @{index_ML Rule_Insts.res_inst_tac: "Proof.context ->
-    ((indexname * Position.T) * string) list -> thm -> int -> tactic"} \\
+    ((indexname * Position.T) * string) list -> (binding * string option * mixfix) list ->
+    thm -> int -> tactic"} \\
   @{index_ML Rule_Insts.eres_inst_tac: "Proof.context ->
-    ((indexname * Position.T) * string) list -> thm -> int -> tactic"} \\
+    ((indexname * Position.T) * string) list -> (binding * string option * mixfix) list ->
+    thm -> int -> tactic"} \\
   @{index_ML Rule_Insts.dres_inst_tac: "Proof.context ->
-    ((indexname * Position.T) * string) list -> thm -> int -> tactic"} \\
+    ((indexname * Position.T) * string) list -> (binding * string option * mixfix) list ->
+    thm -> int -> tactic"} \\
   @{index_ML Rule_Insts.forw_inst_tac: "Proof.context ->
-    ((indexname * Position.T) * string) list -> thm -> int -> tactic"} \\
-  @{index_ML Rule_Insts.subgoal_tac: "Proof.context -> string -> int -> tactic"} \\
-  @{index_ML Rule_Insts.thin_tac: "Proof.context -> string -> int -> tactic"} \\
+    ((indexname * Position.T) * string) list -> (binding * string option * mixfix) list ->
+    thm -> int -> tactic"} \\
+  @{index_ML Rule_Insts.subgoal_tac: "Proof.context -> string ->
+    (binding * string option * mixfix) list -> int -> tactic"} \\
+  @{index_ML Rule_Insts.thin_tac: "Proof.context -> string ->
+    (binding * string option * mixfix) list -> int -> tactic"} \\
   @{index_ML rename_tac: "string list -> int -> tactic"} \\
   \end{mldecls}