--- a/doc-src/IsarImplementation/Thy/Logic.thy Wed Apr 14 11:11:23 2010 +0200
+++ b/doc-src/IsarImplementation/Thy/Logic.thy Wed Apr 14 11:24:31 2010 +0200
@@ -552,10 +552,10 @@
@{index_ML Thm.implies_elim: "thm -> thm -> thm"} \\
@{index_ML Thm.generalize: "string list * string list -> int -> thm -> thm"} \\
@{index_ML Thm.instantiate: "(ctyp * ctyp) list * (cterm * cterm) list -> thm -> thm"} \\
- @{index_ML Thm.add_axiom: "binding * term -> theory -> thm * theory"} \\
+ @{index_ML Thm.add_axiom: "binding * term -> theory -> (string * thm) * theory"} \\
@{index_ML Thm.add_oracle: "binding * ('a -> cterm) -> theory
-> (string * ('a -> thm)) * theory"} \\
- @{index_ML Thm.add_def: "bool -> bool -> binding * term -> theory -> thm * theory"} \\
+ @{index_ML Thm.add_def: "bool -> bool -> binding * term -> theory -> (string * thm) * theory"} \\
\end{mldecls}
\begin{mldecls}
@{index_ML Theory.add_deps: "string -> string * typ -> (string * typ) list -> theory -> theory"} \\