removed tracing output
authorblanchet
Thu, 13 Mar 2014 13:18:13 +0100
changeset 56080 f8ed378ec457
parent 56079 175ac95720d4
child 56081 72fad75baf7e
removed tracing output
src/HOL/Tools/SMT2/z3_new_proof_replay.ML
--- a/src/HOL/Tools/SMT2/z3_new_proof_replay.ML	Thu Mar 13 13:18:13 2014 +0100
+++ b/src/HOL/Tools/SMT2/z3_new_proof_replay.ML	Thu Mar 13 13:18:13 2014 +0100
@@ -55,7 +55,6 @@
 
 fun replay_thm ctxt assumed nthms
     (Z3_New_Proof.Z3_Step {id, rule, concl, fixes, is_fix_step, ...}) =
-(tracing ("replay_thm: " ^ @{make_string} (id, rule) ^ " " ^ Syntax.string_of_term ctxt concl);
   if Z3_New_Proof_Methods.is_assumption rule then
     (case Inttab.lookup assumed id of
       SOME (_, thm) => thm
@@ -63,7 +62,6 @@
   else
     under_fixes (Z3_New_Proof_Methods.method_for rule) ctxt
       (if is_fix_step then (map snd nthms, []) else ([], nthms)) fixes concl
-) (*###*)
 
 fun replay_step ctxt assumed (step as Z3_New_Proof.Z3_Step {id, prems, fixes, ...}) proofs =
   let val nthms = map (the o Inttab.lookup proofs) prems