src/HOL/Tools/Sledgehammer/sledgehammer_fact_minimize.ML
changeset 38696 4c6b65d6a135
parent 38617 f7b32911340b
child 38698 d19c3a7ce38b
equal deleted inserted replaced
38695:e85ce10cef1a 38696:4c6b65d6a135
   155   end
   155   end
   156 
   156 
   157 fun run_minimize params i refs state =
   157 fun run_minimize params i refs state =
   158   let
   158   let
   159     val ctxt = Proof.context_of state
   159     val ctxt = Proof.context_of state
       
   160     val reserved = reserved_isar_keyword_table ()
   160     val chained_ths = #facts (Proof.goal state)
   161     val chained_ths = #facts (Proof.goal state)
   161     val name_thms_pairs = map (name_thms_pair_from_ref ctxt chained_ths) refs
   162     val name_thms_pairs =
       
   163       map (name_thms_pair_from_ref ctxt reserved chained_ths) refs
   162   in
   164   in
   163     case subgoal_count state of
   165     case subgoal_count state of
   164       0 => priority "No subgoal!"
   166       0 => priority "No subgoal!"
   165     | n =>
   167     | n =>
   166       (kill_atps ();
   168       (kill_atps ();