diff -r 7829d6435c60 -r c2ee8d993d6a src/HOL/Tools/SMT/smt_normalize.ML --- a/src/HOL/Tools/SMT/smt_normalize.ML Thu Sep 09 23:07:02 2021 +0200 +++ b/src/HOL/Tools/SMT/smt_normalize.ML Fri Sep 10 14:59:19 2021 +0200 @@ -35,7 +35,7 @@ fun inst f ct thm = let val cv = f (Drule.strip_imp_concl (Thm.cprop_of thm)) - in Thm.instantiate ([], [(dest_Var (Thm.term_of cv), ct)]) thm end + in Thm.instantiate (TVars.empty, Vars.make [(dest_Var (Thm.term_of cv), ct)]) thm end in fun instantiate_elim thm = @@ -203,7 +203,7 @@ let val (ctr, cp) = Thm.dest_binop (Thm.rhs_of trigger_eq) ||> rpair ct val inst = map (apfst (dest_Var o Thm.term_of)) [cp, (ctr, mk_trigger ctss)] - in Thm.instantiate ([], inst) trigger_eq end + in Thm.instantiate (TVars.empty, Vars.make inst) trigger_eq end fun infer_trigger_eq_conv outer_ctxt (ctxt, cvs) ct = let @@ -402,7 +402,7 @@ let val (q, cts) = fold (add_apps add_int_of_nat [] o Thm.cprop_of) thms (false, []) in if q then (thms, nat_int_thms) - else (thms, map (fn ct => Thm.instantiate ([], [(var, ct)]) int_thm) cts) + else (thms, map (fn ct => Thm.instantiate (TVars.empty, Vars.make [(var, ct)]) int_thm) cts) end val setup_nat_as_int =