src/HOL/Tools/SMT/smt_solver.ML
changeset 40199 2963511e121c
parent 40198 8d470bbaafd7
child 40276 6efa052b9213
equal deleted inserted replaced
40198:8d470bbaafd7 40199:2963511e121c
   421   then raise SMT (Other_Failure "proof state contains the universal sort {}")
   421   then raise SMT (Other_Failure "proof state contains the universal sort {}")
   422   else solver_of (Context.Proof ctxt) rm ctxt irules
   422   else solver_of (Context.Proof ctxt) rm ctxt irules
   423 
   423 
   424 fun smt_filter run_remote time_limit st xrules i =
   424 fun smt_filter run_remote time_limit st xrules i =
   425   let
   425   let
   426     val {context, facts, goal} = Proof.goal st
   426     val {facts, goal, ...} = Proof.goal st
   427     val ctxt =
   427     val ctxt =
   428       context
   428       Proof.context_of st
   429       |> Config.put timeout (Time.toSeconds time_limit)
   429       |> Config.put timeout (Time.toSeconds time_limit)
   430       |> Config.put oracle false
   430       |> Config.put oracle false
   431       |> Config.put filter_only true
   431       |> Config.put filter_only true
   432     val cprop =
   432     val cprop =
   433       Thm.cprem_of goal i
   433       Thm.cprem_of goal i