src/HOL/Tools/SMT/smt_solver.ML
changeset 40560 b57f7fee72ee
parent 40550 f84c664ece8e
child 40561 0125cbb5d3c7
equal deleted inserted replaced
40558:e75614d0a859 40560:b57f7fee72ee
   306   let
   306   let
   307     val {facts, goal, ...} = Proof.goal st
   307     val {facts, goal, ...} = Proof.goal st
   308     val ctxt =
   308     val ctxt =
   309       Proof.context_of st
   309       Proof.context_of st
   310       |> Config.put C.oracle false
   310       |> Config.put C.oracle false
   311       |> Config.put C.timeout (Real.fromInt (Time.toSeconds time_limit))
   311       |> Config.put C.timeout (Time.toReal time_limit)
   312       |> Config.put C.drop_bad_facts true
   312       |> Config.put C.drop_bad_facts true
   313       |> Config.put C.filter_only_facts true
   313       |> Config.put C.filter_only_facts true
   314     val ({context=ctxt', prems, concl, ...}, _) = Subgoal.focus ctxt i goal
   314     val ({context=ctxt', prems, concl, ...}, _) = Subgoal.focus ctxt i goal
   315     val cprop =
   315     val cprop =
   316       concl
   316       concl