src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML
changeset 64413 c0d5e78eb647
parent 63337 ae9330fdbc16
child 65458 cf504b7a7aa7
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML	Wed Oct 26 20:59:36 2016 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML	Wed Oct 26 22:40:28 2016 +0200
@@ -458,7 +458,7 @@
 fun all_facts ctxt generous ho_atp keywords add_ths chained css =
   let
     val thy = Proof_Context.theory_of ctxt
-    val transfer = Global_Theory.transfer_theories thy;
+    val transfer = Global_Theory.transfer_theories thy
     val global_facts = Global_Theory.facts_of thy
     val is_too_complex =
       if generous orelse fact_count global_facts >= max_facts_for_complex_check then K false
@@ -528,7 +528,7 @@
   in
     (* The single-theorem names go before the multiple-theorem ones (e.g., "xxx" vs. "xxx(3)"), so
        that single names are preferred when both are available. *)
-    `I []
+    ([], [])
     |> add_facts false fold local_facts (unnamed_locals @ named_locals)
     |> add_facts true Facts.fold_static global_facts global_facts
     |> op @