doc-src/IsarImplementation/Thy/proof.thy
changeset 20171 424739228123
parent 20064 92aad017b847
child 20218 be3bfb0699ba
--- a/doc-src/IsarImplementation/Thy/proof.thy	Thu Jul 20 14:34:57 2006 +0200
+++ b/doc-src/IsarImplementation/Thy/proof.thy	Thu Jul 20 14:35:37 2006 +0200
@@ -18,7 +18,6 @@
   @{index_ML Variable.import: "bool -> thm list -> Proof.context -> thm list * Proof.context"} \\
   @{index_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
   @{index_ML Variable.trade: "Proof.context -> (thm list -> thm list) -> thm list -> thm list"} \\
-  @{index_ML Variable.monomorphic: "Proof.context -> term list -> term list"} \\
   @{index_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
   \end{mldecls}
 
@@ -56,9 +55,6 @@
   Variable.export}, i.e.\ it provides a view on facts with all
   variables being fixed in the current context.
 
-  \item @{ML Variable.monomorphic}~@{text "ctxt ts"} introduces fixed
-  type variables for the schematic ones in @{text "ts"}.
-
   \item @{ML Variable.polymorphic}~@{text "ctxt ts"} generalizes type
   variables in @{text "ts"} as far as possible, even those occurring
   in fixed term variables.  This operation essentially reverses the