aboutsummaryrefslogtreecommitdiff
path: root/proofs/refine.ml
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2018-12-05 02:49:07 +0100
committerEmilio Jesus Gallego Arias2018-12-13 13:55:40 +0100
commit1499565d4ef1165d34b5bbb927e52a754903e077 (patch)
tree297d86f152bf2c4d31ae8ab6c819b451f01e6310 /proofs/refine.ml
parent228f0d929bb5098d58cd285fde42bb08d70c6ee8 (diff)
[engine] Allow debug printers to access the environment.
This should improve correctness and will be needed for the PRs that remove global access to the proof state.
Diffstat (limited to 'proofs/refine.ml')
-rw-r--r--proofs/refine.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/proofs/refine.ml b/proofs/refine.ml
index d812a8cad7..1d796fece5 100644
--- a/proofs/refine.ml
+++ b/proofs/refine.ml
@@ -107,8 +107,8 @@ let generic_refine ~typecheck f gl =
(* Mark goals *)
let sigma = Proofview.Unsafe.mark_as_goals sigma comb in
let comb = CList.map (fun x -> Proofview.goal_with_state x state) comb in
- let trace () = Pp.(hov 2 (str"simple refine"++spc()++
- Termops.Internal.print_constr_env env sigma c)) in
+ let trace env sigma = Pp.(hov 2 (str"simple refine"++spc()++
+ Termops.Internal.print_constr_env env sigma c)) in
Proofview.Trace.name_tactic trace (Proofview.tclUNIT v) >>= fun v ->
Proofview.Unsafe.tclSETENV (Environ.reset_context env) <*>
Proofview.Unsafe.tclEVARS sigma <*>