src/HOL/Tools/Sledgehammer/sledgehammer_run.ML
changeset 48299 5e5c6616f0fe
parent 48293 914ca0827804
child 48319 340187063d84
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_run.ML	Wed Jul 18 08:44:03 2012 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_run.ML	Wed Jul 18 08:44:03 2012 +0200
@@ -171,8 +171,11 @@
       val {facts = chained_ths, goal, ...} = Proof.goal state
       val (_, hyp_ts, concl_t) = strip_subgoal ctxt goal i
       val ho_atp = exists (Sledgehammer_Provers.is_ho_atp ctxt) provers
+      val reserved = reserved_isar_keyword_table ()
+      val css_table = clasimpset_rule_table_of ctxt
       val facts =
-        nearly_all_facts ctxt ho_atp fact_override chained_ths hyp_ts concl_t
+        nearly_all_facts ctxt ho_atp fact_override reserved css_table
+                         chained_ths hyp_ts concl_t
       val _ = () |> not blocking ? kill_provers
       val _ = case find_first (not o is_prover_supported ctxt) provers of
                 SOME name => error ("No such prover: " ^ name ^ ".")