doc-src/IsarImplementation/Thy/proof.thy
changeset 20797 c1f0bc7e7d80
parent 20547 796ae7fa1049
child 21827 0b1d07f79c1e
--- a/doc-src/IsarImplementation/Thy/proof.thy	Sat Sep 30 20:54:34 2006 +0200
+++ b/doc-src/IsarImplementation/Thy/proof.thy	Sat Sep 30 21:39:17 2006 +0200
@@ -88,7 +88,7 @@
   \begin{mldecls}
   @{index_ML Variable.add_fixes: "
   string list -> Proof.context -> string list * Proof.context"} \\
-  @{index_ML Variable.invent_fixes: "
+  @{index_ML Variable.variant_fixes: "
   string list -> Proof.context -> string list * Proof.context"} \\
   @{index_ML Variable.declare_term: "term -> Proof.context -> Proof.context"} \\
   @{index_ML Variable.declare_constraints: "term -> Proof.context -> Proof.context"} \\
@@ -108,7 +108,7 @@
   already.  There is a different policy within a local proof body: the
   given names are just hints for newly invented Skolem variables.
 
-  \item @{ML Variable.invent_fixes} is similar to @{ML
+  \item @{ML Variable.variant_fixes} is similar to @{ML
   Variable.add_fixes}, but always produces fresh variants of the given
   names.