src/HOL/Tools/SMT/verit_replay.ML
changeset 72513 75f5c63f6cfa
parent 72459 15fc6320da68
child 75274 e89709b80b6e
equal deleted inserted replaced
72512:83b5911c0164 72513:75f5c63f6cfa
   129 
   129 
   130     (*for sko_ex and sko_forall, assumptions are in proofs',  but the definition of the skolem
   130     (*for sko_ex and sko_forall, assumptions are in proofs',  but the definition of the skolem
   131        function is in proofs *)
   131        function is in proofs *)
   132     val nthms = prems
   132     val nthms = prems
   133       |> map (apsnd export_thm) o map_filter (Symtab.lookup (if (null subproof) then proofs else proofs'))
   133       |> map (apsnd export_thm) o map_filter (Symtab.lookup (if (null subproof) then proofs else proofs'))
   134     val nthms' = (if Verit_Proof.is_skolemisation rule
   134     val nthms' = (if Verit_Proof.is_skolemization rule
   135          then prems else [])
   135          then prems else [])
   136       |> map_filter (Symtab.lookup proofs)
   136       |> map_filter (Symtab.lookup proofs)
   137     val args = map (Term.subst_free concl_tranformation o subst_only_free global_transformation) args
   137     val args = map (Term.subst_free concl_tranformation o subst_only_free global_transformation) args
   138     val insts = Symtab.map (K (Term.subst_free concl_tranformation o subst_only_free global_transformation)) insts
   138     val insts = Symtab.map (K (Term.subst_free concl_tranformation o subst_only_free global_transformation)) insts
   139     val proof_prems =
   139     val proof_prems =