src/HOL/Tools/TFL/post.ML
changeset 55236 8d61b0aa7a0d
parent 55151 f331472f1027
child 56245 84fc7dfa3cd4
--- a/src/HOL/Tools/TFL/post.ML	Sat Feb 01 18:41:48 2014 +0100
+++ b/src/HOL/Tools/TFL/post.ML	Sat Feb 01 18:42:46 2014 +0100
@@ -101,14 +101,12 @@
                      if (solved th) then (th::So, Si, St)
                      else (So, th::Si, St)) nested_tcs ([],[],[])
               val simplified' = map (join_assums ctxt) simplified
-              val dummy = (Prim.trace_thms "solved =" solved;
-                           Prim.trace_thms "simplified' =" simplified')
+              val dummy = (Prim.trace_thms ctxt "solved =" solved;
+                           Prim.trace_thms ctxt "simplified' =" simplified')
               val rewr = full_simplify (ctxt addsimps (solved @ simplified'));
-              val dummy = Prim.trace_thms "Simplifying the induction rule..."
-                                          [induction]
+              val dummy = Prim.trace_thms ctxt "Simplifying the induction rule..." [induction]
               val induction' = rewr induction
-              val dummy = Prim.trace_thms "Simplifying the recursion rules..."
-                                          [rules]
+              val dummy = Prim.trace_thms ctxt "Simplifying the recursion rules..." [rules]
               val rules'     = rewr rules
               val _ = writeln "... Postprocessing finished";
           in
@@ -142,7 +140,7 @@
            Prim.post_definition congs thy ctxt (def, pats)
        val {lhs=f,rhs} = USyntax.dest_eq (concl def)
        val (_,[R,_]) = USyntax.strip_comb rhs
-       val dummy = Prim.trace_thms "congs =" congs
+       val dummy = Prim.trace_thms ctxt "congs =" congs
        (*the next step has caused simplifier looping in some cases*)
        val {induction, rules, tcs} =
              proof_stage strict ctxt wfs thy