src/Pure/Isar/element.ML
changeset 74282 c2ee8d993d6a
parent 71018 d32ed8927a42
child 74509 f24ade4ff3cc
--- a/src/Pure/Isar/element.ML	Thu Sep 09 23:07:02 2021 +0200
+++ b/src/Pure/Isar/element.ML	Fri Sep 10 14:59:19 2021 +0200
@@ -47,8 +47,7 @@
   val transform_witness: morphism -> witness -> witness
   val conclude_witness: Proof.context -> witness -> thm
   val pretty_witness: Proof.context -> witness -> Pretty.T
-  val instantiate_normalize_morphism:
-    ((string * sort) * ctyp) list * ((string * typ) * cterm) list -> morphism
+  val instantiate_normalize_morphism: ctyp TFrees.table * cterm Frees.table -> morphism
   val satisfy_morphism: witness list -> morphism
   val eq_term_morphism: theory -> term list -> morphism option
   val eq_morphism: theory -> thm list -> morphism option
@@ -208,7 +207,8 @@
     SOME C =>
       let
         val thesis = Var ((Auto_Bind.thesisN, Thm.maxidx_of th + 1), fastype_of C);
-        val th' = Thm.instantiate ([], [(Term.dest_Var C, Thm.cterm_of ctxt thesis)]) th;
+        val insts = (TVars.empty, Vars.make [(Term.dest_Var C, Thm.cterm_of ctxt thesis)]);
+        val th' = Thm.instantiate insts th;
       in (th', true) end
   | NONE => (th, false));