aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--ide/richprinter.ml1
-rw-r--r--ide/texmacspp.ml4
-rw-r--r--tactics/tactics.ml6
3 files changed, 5 insertions, 6 deletions
diff --git a/ide/richprinter.ml b/ide/richprinter.ml
index 5f39f36ea..995cef1ac 100644
--- a/ide/richprinter.ml
+++ b/ide/richprinter.ml
@@ -2,7 +2,6 @@ open Richpp
module RichppConstr = Ppconstr.Richpp
module RichppVernac = Ppvernac.Richpp
-module RichppTactic = Pptactic.Richpp
type rich_pp =
Ppannotation.t Richpp.located Xml_datatype.gxml
diff --git a/ide/texmacspp.ml b/ide/texmacspp.ml
index 458e84835..328ddd0cd 100644
--- a/ide/texmacspp.ml
+++ b/ide/texmacspp.ml
@@ -127,10 +127,6 @@ let xmlProofMode loc name = xmlWithLoc loc "proofmode" ["name",name] []
let xmlProof loc xml = xmlWithLoc loc "proof" [] xml
-let xmlRawTactic name rtac =
- Element("rawtactic", ["name",name],
- [PCData (Pp.string_of_ppcmds (Pptactic.pr_raw_tactic rtac))])
-
let xmlSectionSubsetDescr name ssd =
Element("sectionsubsetdescr",["name",name],
[PCData (Proof_using.to_string ssd)])
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