diff -r 36497ee02ed8 -r 4970437fe092 src/Doc/IsarImplementation/Tactic.thy --- a/src/Doc/IsarImplementation/Tactic.thy Thu Jun 27 11:07:48 2013 +0200 +++ b/src/Doc/IsarImplementation/Tactic.thy Thu Jun 27 11:33:42 2013 +0200 @@ -491,7 +491,7 @@ text %mlref {* \begin{mldecls} @{index_ML compose_tac: "(bool * thm * int) -> int -> tactic"} \\ - @{index_ML compose: "thm * int * thm -> thm list"} \\ + @{index_ML Drule.compose: "thm * int * thm -> thm list"} \\ @{index_ML_op COMP: "thm * thm -> thm"} \\ \end{mldecls} @@ -505,14 +505,14 @@ performs elim-resolution --- it solves the first premise of @{text "rule"} by assumption and deletes that assumption. - \item @{ML compose}~@{text "(thm\<^sub>1, i, thm\<^sub>2)"} uses @{text "thm\<^sub>1"}, + \item @{ML Drule.compose}~@{text "(thm\<^sub>1, i, thm\<^sub>2)"} uses @{text "thm\<^sub>1"}, regarded as an atomic formula, to solve premise @{text "i"} of @{text "thm\<^sub>2"}. Let @{text "thm\<^sub>1"} and @{text "thm\<^sub>2"} be @{text "\"} and @{text "\\<^sub>1 \ \ \\<^sub>n \ \"}. For each @{text "s"} that unifies @{text "\"} and @{text "\"}, the result list contains the theorem @{text "(\\<^sub>1 \ \ \\<^sub>i\<^sub>-\<^sub>1 \ \\<^sub>i\<^sub>+\<^sub>1 \ \ \\<^sub>n \ \)s"}. - \item @{text "thm\<^sub>1 COMP thm\<^sub>2"} calls @{text "compose (thm\<^sub>1, 1, + \item @{text "thm\<^sub>1 COMP thm\<^sub>2"} calls @{text "Drule.compose (thm\<^sub>1, 1, thm\<^sub>2)"} and returns the result, if unique; otherwise, it raises exception @{ML THM}.