src/HOL/Tools/Sledgehammer/sledgehammer_run.ML
changeset 52196 2281f33e8da6
parent 52125 ac7830871177
child 52555 6811291d1869
equal deleted inserted replaced
52195:056ec8201667 52196:2281f33e8da6
   196       val print = if mode = Normal then Output.urgent_message else K ()
   196       val print = if mode = Normal then Output.urgent_message else K ()
   197       val state =
   197       val state =
   198         state |> Proof.map_context (Config.put SMT_Config.verbose debug)
   198         state |> Proof.map_context (Config.put SMT_Config.verbose debug)
   199       val ctxt = Proof.context_of state
   199       val ctxt = Proof.context_of state
   200       val {facts = chained, goal, ...} = Proof.goal state
   200       val {facts = chained, goal, ...} = Proof.goal state
   201       val ((_, hyp_ts, concl_t), _) = strip_subgoal goal i ctxt
   201       val (_, hyp_ts, concl_t) = strip_subgoal goal i ctxt
   202       val ho_atp = exists (is_ho_atp ctxt) provers
   202       val ho_atp = exists (is_ho_atp ctxt) provers
   203       val reserved = reserved_isar_keyword_table ()
   203       val reserved = reserved_isar_keyword_table ()
   204       val css = clasimpset_rule_table_of ctxt
   204       val css = clasimpset_rule_table_of ctxt
   205       val all_facts =
   205       val all_facts =
   206         nearly_all_facts ctxt ho_atp fact_override reserved css chained hyp_ts
   206         nearly_all_facts ctxt ho_atp fact_override reserved css chained hyp_ts