aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-09-09 00:47:46 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-09-09 00:54:09 +0200
commita6cd6948fa592f21b67916f423fe2adb62085492 (patch)
treecb4783153f70f6ff3fd3aeb1cf237d0912e59eb5 /tactics
parent7045848145c16d978456aab2edd192c54d242e69 (diff)
Removing the last uses of Pptactic in the lower layers.
Diffstat (limited to 'tactics')
-rw-r--r--tactics/tactics.ml6
1 files changed, 5 insertions, 1 deletions
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 85b6e8de9..cae45f607 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -871,7 +871,11 @@ let reduction_clause redexp cl =
(None, bind_red_expr_occurrences occs nbcl redexp)) cl
let reduce redexp cl =
- let trace () = Pp.(hov 2 (Pptactic.pr_atomic_tactic (Global.env()) (TacReduce (redexp,cl)))) in
+ let trace () =
+ let open Printer in
+ let pr = (pr_constr, pr_lconstr, pr_evaluable_reference, pr_constr_pattern) in
+ Pp.(hov 2 (Pputils.pr_red_expr pr str redexp))
+ in
Proofview.Trace.name_tactic trace begin
Proofview.Goal.enter { enter = begin fun gl ->
let cl' = concrete_clause_of (fun () -> Tacmach.New.pf_ids_of_hyps gl) cl in