src/HOL/Tools/Sledgehammer/sledgehammer_filter.ML
changeset 42361 23f352990944
parent 42358 b47d41d9f4b5
child 42449 494e4ac5b0f8
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_filter.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_filter.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -199,7 +199,7 @@
 fun instantiate_if_induct_rule ctxt stmt stmt_xs (ax as (_, (_, th))) =
   case struct_induct_rule_on th of
     SOME (p_name, ind_T) =>
-    let val thy = ProofContext.theory_of ctxt in
+    let val thy = Proof_Context.theory_of ctxt in
       stmt_xs |> filter (fn (_, T) => type_match thy (T, ind_T))
               |> map_filter (try (instantiate_induct_rule ctxt stmt p_name ax))
     end
@@ -542,7 +542,7 @@
         (fudge as {threshold_divisor, ridiculous_threshold, ...})
         ({add, del, ...} : relevance_override) facts goal_ts =
   let
-    val thy = ProofContext.theory_of ctxt
+    val thy = Proof_Context.theory_of ctxt
     val const_tab = fold (count_fact_consts thy fudge) facts Symtab.empty
     val goal_const_tab =
       pconsts_in_terms thy is_built_in_const false (SOME false) goal_ts
@@ -797,9 +797,9 @@
               ({intro_bonus, elim_bonus, simp_bonus, ...} : relevance_fudge)
               add_ths chained_ths =
   let
-    val thy = ProofContext.theory_of ctxt
+    val thy = Proof_Context.theory_of ctxt
     val global_facts = Global_Theory.facts_of thy
-    val local_facts = ProofContext.facts_of ctxt
+    val local_facts = Proof_Context.facts_of ctxt
     val named_locals = local_facts |> Facts.dest_static []
     val assms = Assumption.all_assms_of ctxt
     fun is_assum th = exists (fn ct => prop_of th aconv term_of ct) assms
@@ -832,7 +832,7 @@
             val backquote_thm =
               backquote o string_for_term ctxt o close_form o prop_of
             fun check_thms a =
-              case try (ProofContext.get_thms ctxt) a of
+              case try (Proof_Context.get_thms ctxt) a of
                 NONE => false
               | SOME ths' => Thm.eq_thms (ths, ths')
           in
@@ -887,7 +887,7 @@
                    max_relevant is_built_in_const fudge
                    (override as {add, only, ...}) chained_ths hyp_ts concl_t =
   let
-    val thy = ProofContext.theory_of ctxt
+    val thy = Proof_Context.theory_of ctxt
     val decay = Math.pow ((1.0 - threshold1) / (1.0 - threshold0),
                           1.0 / Real.fromInt (max_relevant + 1))
     val add_ths = Attrib.eval_thms ctxt add