aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.ml
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-09-01 09:59:20 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-09-01 10:00:47 +0200
commit18046e2525300b990db4c8817f1cc02dcab97445 (patch)
treec8e7109616e252ebecedc42097ddae6f6ed15751 /tactics/tactics.ml
parent7d4b8108bc8fa6951e605cb9b42580ff6f8e583f (diff)
Moving log of "TacReduce"/"reduce" to Tactics.reduce so that internal
calls are logged too. Using appropriate printer for reparsability of the output.
Diffstat (limited to 'tactics/tactics.ml')
-rw-r--r--tactics/tactics.ml7
1 files changed, 5 insertions, 2 deletions
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index acc0fa1ca..c9cec828c 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -869,14 +869,17 @@ 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
+ 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
- let redexps = reduction_clause redexp cl in
+ let cl' = concrete_clause_of (fun () -> Tacmach.New.pf_ids_of_hyps gl) cl in
+ let redexps = reduction_clause redexp cl' in
let check = match redexp with Fold _ | Pattern _ -> true | _ -> false in
Tacticals.New.tclMAP (fun (where,redexp) ->
e_reduct_option ~check
(Redexpr.reduction_of_red_expr (Tacmach.New.pf_env gl) redexp) where) redexps
end }
+ end
(* Unfolding occurrences of a constant *)