src/HOL/Probability/measurable.ML
changeset 59498 50b60f501b05
parent 59353 f0707dc3d9aa
child 59582 0fbed69ff081
--- a/src/HOL/Probability/measurable.ML	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/HOL/Probability/measurable.ML	Tue Feb 10 14:48:26 2015 +0100
@@ -208,9 +208,9 @@
     fun r_tac msg =
       if Config.get ctxt debug
       then FIRST' o
-        map (fn thm => resolve_tac [thm]
+        map (fn thm => resolve_tac ctxt [thm]
           THEN' K (debug_tac ctxt (debug_fact (msg ^ " resolved using") thm) all_tac))
-      else resolve_tac
+      else resolve_tac ctxt
 
     val elem_congI = @{lemma "A = B \<Longrightarrow> x \<in> B \<Longrightarrow> x \<in> A" by simp}
 
@@ -249,7 +249,8 @@
           val f = dest_measurable_fun (HOLogic.dest_Trueprop t)
           fun cert f = map (Option.map (f (Proof_Context.theory_of ctxt)))
           fun inst (ts, Ts) =
-            Drule.instantiate' (cert ctyp_of Ts) (cert cterm_of ts) @{thm measurable_compose_countable}
+            Drule.instantiate' (cert ctyp_of Ts) (cert cterm_of ts)
+              @{thm measurable_compose_countable}
         in r_tac "split countable" (cnt_prefixes ctxt f |> map inst) i end
         handle TERM _ => no_tac) 1)