src/HOL/Tools/Nitpick/nitpick.ML
changeset 73386 3fb201ca8fb5
parent 72329 6255e532aa36
child 73387 3b5196dac4c8
--- a/src/HOL/Tools/Nitpick/nitpick.ML	Fri Mar 05 16:45:16 2021 +0100
+++ b/src/HOL/Tools/Nitpick/nitpick.ML	Fri Mar 05 17:02:32 2021 +0100
@@ -201,7 +201,6 @@
                            subst def_assm_ts nondef_assm_ts orig_t =
   let
     val time_start = Time.now ()
-    val timer = Timer.startRealTimer ()
     val thy = Proof.theory_of state
     val ctxt = Proof.context_of state
     val keywords = Thy_Header.get_keywords thy
@@ -933,8 +932,7 @@
       handle Timeout.TIMEOUT _ =>
              (print_nt (fn () => excipit "ran out of time after checking");
               if !met_potential > 0 then potentialN else unknownN)
-    val _ = print_v (fn () =>
-                "Total time: " ^ string_of_time (Timer.checkRealTimer timer))
+    val _ = print_v (fn () => "Total time: " ^ string_of_time (Time.now () - time_start))
     val _ = spying spy (fn () => (state, i, "outcome: " ^ outcome_code))
   in (outcome_code, Queue.content (Synchronized.value outcome)) end