src/HOL/Tools/Sledgehammer/sledgehammer_mepo.ML
changeset 54142 5f3c1b445253
parent 54124 d3c0cf737b55
child 54143 18def1c73c79
equal deleted inserted replaced
54141:f57f8e7a879f 54142:5f3c1b445253
   437 
   437 
   438 fun relevance_filter ctxt thres0 decay max_facts
   438 fun relevance_filter ctxt thres0 decay max_facts
   439         (fudge as {threshold_divisor, ridiculous_threshold, ...}) facts hyp_ts concl_t =
   439         (fudge as {threshold_divisor, ridiculous_threshold, ...}) facts hyp_ts concl_t =
   440   let
   440   let
   441     val thy = Proof_Context.theory_of ctxt
   441     val thy = Proof_Context.theory_of ctxt
   442     val facts = drop_duplicate_facts thy facts
   442     val facts = drop_duplicate_facts facts
   443     val const_tab = fold (count_fact_consts thy fudge) facts Symtab.empty
   443     val const_tab = fold (count_fact_consts thy fudge) facts Symtab.empty
   444     val add_pconsts = add_pconsts_in_term thy
   444     val add_pconsts = add_pconsts_in_term thy
   445     val chained_ts =
   445     val chained_ts =
   446       facts |> map_filter (fn ((_, (Chained, _)), th) => SOME (prop_of th)
   446       facts |> map_filter (fn ((_, (Chained, _)), th) => SOME (prop_of th)
   447                             | _ => NONE)
   447                             | _ => NONE)