aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2016-06-14 12:02:40 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2016-06-14 12:02:40 +0200
commit494312f05a10188cf51f66cf189681f389e179b2 (patch)
treef29e7ea7903ee14d02ffc06c29444ce0e50747b8 /toplevel
parent2b19f0923a314a6df0a9cfed0f56cf2405e6591c (diff)
parent4ae315f92e4a9849a56d3d9b0da33027f362d6e8 (diff)
Merge branch 'bug4725' into v8.5
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/command.ml1
-rw-r--r--toplevel/obligations.ml6
2 files changed, 0 insertions, 7 deletions
diff --git a/toplevel/command.ml b/toplevel/command.ml
index 8f7c38997..8eb2232ed 100644
--- a/toplevel/command.ml
+++ b/toplevel/command.ml
@@ -923,7 +923,6 @@ let build_wellfounded (recname,pl,n,bl,arityc,body) poly r measure notation =
let binders = letbinders @ [arg] in
let binders_env = push_rel_context binders_rel env in
let rel, _ = interp_constr_evars_impls env evdref r in
- let () = check_evars_are_solved env !evdref (Evd.empty,!evdref) in
let relty = Typing.unsafe_type_of env !evdref rel in
let relargty =
let error () =
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