src/HOL/TPTP/TPTP_Proof_Reconstruction.thy
changeset 74282 c2ee8d993d6a
parent 69605 a96320074298
child 77879 dd222e2af01a
--- a/src/HOL/TPTP/TPTP_Proof_Reconstruction.thy	Thu Sep 09 23:07:02 2021 +0200
+++ b/src/HOL/TPTP/TPTP_Proof_Reconstruction.thy	Fri Sep 10 14:59:19 2021 +0200
@@ -943,7 +943,7 @@
      end
 
     fun instantiate_tac from to =
-      PRIMITIVE (Thm.instantiate ([], [(from, to)]))
+      PRIMITIVE (Thm.instantiate (TVars.empty, Vars.make [(from, to)]))
 
     val tactic =
       if is_none var_opt then no_tac