src/HOL/Tools/Sledgehammer/sledgehammer_filter.ML
changeset 40408 0d0acdf068b8
parent 40375 db690d38e4b9
child 40418 8b73059e97a1
equal deleted inserted replaced
40388:cb9fd7dd641c 40408:0d0acdf068b8
   518     fun add_add_ths accepts =
   518     fun add_add_ths accepts =
   519       (facts |> filter ((member Thm.eq_thm add_ths
   519       (facts |> filter ((member Thm.eq_thm add_ths
   520                          andf (not o member (Thm.eq_thm o apsnd snd) accepts))
   520                          andf (not o member (Thm.eq_thm o apsnd snd) accepts))
   521                         o snd))
   521                         o snd))
   522       @ accepts
   522       @ accepts
       
   523       |> take max_relevant
   523   in
   524   in
   524     facts |> map_filter (pair_consts_fact thy is_built_in_const fudge)
   525     facts |> map_filter (pair_consts_fact thy is_built_in_const fudge)
   525           |> iter 0 max_relevant threshold0 goal_const_tab []
   526           |> iter 0 max_relevant threshold0 goal_const_tab []
   526           |> not (null add_ths) ? add_add_ths
   527           |> not (null add_ths) ? add_add_ths
   527           |> tap (fn res => trace_msg (fn () =>
   528           |> tap (fn res => trace_msg (fn () =>