changeset 77879 | dd222e2af01a |
parent 74282 | c2ee8d993d6a |
child 78727 | 1b052426a2b7 |
--- a/src/HOL/TPTP/TPTP_Proof_Reconstruction.thy Tue Apr 18 21:47:40 2023 +0200 +++ b/src/HOL/TPTP/TPTP_Proof_Reconstruction.thy Tue Apr 18 22:24:48 2023 +0200 @@ -943,7 +943,7 @@ end fun instantiate_tac from to = - PRIMITIVE (Thm.instantiate (TVars.empty, Vars.make [(from, to)])) + PRIMITIVE (Thm.instantiate (TVars.empty, Vars.make1 (from, to))) val tactic = if is_none var_opt then no_tac