src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML
changeset 56158 c2c6d560e7b2
parent 56141 c06202417c4a
child 56245 84fc7dfa3cd4
equal deleted inserted replaced
56157:7cfe7b6d501a 56158:c2c6d560e7b2
   457          fact_count global_facts >= max_facts_for_complex_check then
   457          fact_count global_facts >= max_facts_for_complex_check then
   458         K false
   458         K false
   459       else
   459       else
   460         is_too_complex
   460         is_too_complex
   461     val local_facts = Proof_Context.facts_of ctxt
   461     val local_facts = Proof_Context.facts_of ctxt
   462     val named_locals = local_facts |> Facts.dest_static [global_facts]
   462     val named_locals = local_facts |> Facts.dest_static true [global_facts]
   463     val assms = Assumption.all_assms_of ctxt
   463     val assms = Assumption.all_assms_of ctxt
   464     fun is_good_unnamed_local th =
   464     fun is_good_unnamed_local th =
   465       not (Thm.has_name_hint th) andalso
   465       not (Thm.has_name_hint th) andalso
   466       forall (fn (_, ths) => not (member Thm.eq_thm_prop ths th)) named_locals
   466       forall (fn (_, ths) => not (member Thm.eq_thm_prop ths th)) named_locals
   467     val unnamed_locals =
   467     val unnamed_locals =