src/Doc/Implementation/Proof.thy
changeset 60642 48dd1cefb4ae
parent 59902 6afbe5a99139
child 60695 757549b4bbe6
--- a/src/Doc/Implementation/Proof.thy	Fri Jul 03 16:19:45 2015 +0200
+++ b/src/Doc/Implementation/Proof.thy	Sun Jul 05 15:02:30 2015 +0200
@@ -108,7 +108,7 @@
   @{index_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
   @{index_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
   @{index_ML Variable.import: "bool -> thm list -> Proof.context ->
-  (((ctyp * ctyp) list * (cterm * cterm) list) * thm list) * Proof.context"} \\
+  ((((indexname * sort) * ctyp) list * ((indexname * typ) * cterm) list) * thm list) * Proof.context"} \\
   @{index_ML Variable.focus: "term -> Proof.context ->
   ((string * (string * typ)) list * term) * Proof.context"} \\
   \end{mldecls}