aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2016-05-26 10:18:10 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2016-05-26 11:01:28 +0200
commit62fa31d219dcf2129c55b3c46b8cc25be60edcab (patch)
tree0d80cb1d1a2a18702ec7aecfcf2779d6da2fa3b3 /toplevel
parent891a8a9f7ea3bb5b0b07dc5a2df51314135d8b53 (diff)
Program: remove debug tracing
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/obligations.ml6
1 files changed, 0 insertions, 6 deletions
diff --git a/toplevel/obligations.ml b/toplevel/obligations.ml
index a18552c5e..6f7a5f684 100644
--- a/toplevel/obligations.ml
+++ b/toplevel/obligations.ml
@@ -24,10 +24,6 @@ open Util
let declare_fix_ref = ref (fun ?opaque _ _ _ _ _ _ -> assert false)
let declare_definition_ref = ref (fun _ _ _ _ _ -> assert false)
-let trace s =
- if !Flags.debug then msg_debug s
- else ()
-
let succfix (depth, fixrels) =
(succ depth, List.map succ fixrels)
@@ -871,8 +867,6 @@ let rec solve_obligation prg num tac =
let auto n tac oblset = auto_solve_obligations n ~oblset tac in
let hook ctx = Lemmas.mk_hook (obligation_hook prg obl num auto ctx) in
let () = Lemmas.start_proof_univs ~sign:prg.prg_sign obl.obl_name kind evd obl.obl_type hook in
- let () = trace (str "Started obligation " ++ int user_num ++ str " proof: " ++
- Printer.pr_constr_env (Global.env ()) Evd.empty obl.obl_type) in
let _ = Pfedit.by (snd (get_default_tactic ())) in
Option.iter (fun tac -> Pfedit.set_end_tac tac) tac