aboutsummaryrefslogtreecommitdiffhomepage
path: root/ltac/tacinterp.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 /ltac/tacinterp.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 'ltac/tacinterp.ml')
-rw-r--r--ltac/tacinterp.ml3
1 files changed, 0 insertions, 3 deletions
diff --git a/ltac/tacinterp.ml b/ltac/tacinterp.ml
index 397cd988d..83d67c8e3 100644
--- a/ltac/tacinterp.ml
+++ b/ltac/tacinterp.ml
@@ -1822,13 +1822,10 @@ and interp_atomic ist tac : unit Proofview.tactic =
(* Conversion *)
| TacReduce (r,cl) ->
- (* spiwack: until the tactic is in the monad *)
- Proofview.Trace.name_tactic (fun () -> Pp.str"<reduce>") begin
Proofview.Goal.nf_s_enter { s_enter = begin fun gl ->
let (sigma,r_interp) = interp_red_expr ist (pf_env gl) (project gl) r in
Sigma.Unsafe.of_pair (Tactics.reduce r_interp (interp_clause ist (pf_env gl) (project gl) cl), sigma)
end }
- end
| TacChange (None,c,cl) ->
(* spiwack: until the tactic is in the monad *)
Proofview.Trace.name_tactic (fun () -> Pp.str"<change>") begin