src/HOL/Tools/Sledgehammer/sledgehammer_prover_minimize.ML
changeset 58085 ee65e9cfe284
parent 58061 3d060f43accb
child 58494 ed380b9594b5
equal deleted inserted replaced
58084:9f77084444df 58085:ee65e9cfe284
   189 
   189 
   190 fun minimize_facts do_learn prover_name (params as {learn, timeout, ...}) silent i n state goal
   190 fun minimize_facts do_learn prover_name (params as {learn, timeout, ...}) silent i n state goal
   191     facts =
   191     facts =
   192   let
   192   let
   193     val ctxt = Proof.context_of state
   193     val ctxt = Proof.context_of state
   194     val prover = get_prover ctxt (if silent then Auto_Minimize else Minimize) prover_name
   194     val prover = get_prover ctxt Minimize prover_name
   195     fun test timeout = test_facts params silent prover timeout i n state goal
   195     fun test timeout = test_facts params silent prover timeout i n state goal
   196     val (chained, non_chained) = List.partition is_fact_chained facts
   196     val (chained, non_chained) = List.partition is_fact_chained facts
   197     (* Push chained facts to the back, so that they are less likely to be kicked out by the linear
   197     (* Push chained facts to the back, so that they are less likely to be kicked out by the linear
   198        minimization algorithm. *)
   198        minimization algorithm. *)
   199     val facts = non_chained @ chained
   199     val facts = non_chained @ chained