aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-29 01:18:30 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-29 01:20:55 +0200
commita4458475187de726b1518e536cb1a42e8c9d0534 (patch)
tree8c4f361ff4a7770d86cccf4859c4c669fe23f97b
parentd2bb28988b9424620740c34f4475f0205e0a0f73 (diff)
Fixing #5164 (regression in locating error in argument of "refine").
Reporting location was not expecting a term passed to an ML tactic to be interpreted by the ML tactic itself. Made an empirical fix to report about the as-precise-as-possible location available.
-rw-r--r--ltac/tactic_debug.ml5
1 files changed, 3 insertions, 2 deletions
diff --git a/ltac/tactic_debug.ml b/ltac/tactic_debug.ml
index e1c9fed63..5cbddc7f6 100644
--- a/ltac/tactic_debug.ml
+++ b/ltac/tactic_debug.ml
@@ -385,6 +385,8 @@ let skip_extensions trace =
| [] -> [] in
List.rev (aux (List.rev trace))
+let finer_loc loc1 loc2 = Loc.merge loc1 loc2 = loc2
+
let extract_ltac_trace trace eloc =
let trace = skip_extensions trace in
let (loc,c),tail = List.sep_last trace in
@@ -392,11 +394,10 @@ let extract_ltac_trace trace eloc =
(* We entered a user-defined tactic,
we display the trace with location of the call *)
let msg = hov 0 (explain_ltac_call_trace c tail eloc ++ fnl()) in
- Some msg, loc
+ Some msg, if finer_loc eloc loc then eloc else loc
else
(* We entered a primitive tactic, we don't display trace but
report on the finest location *)
- let finer_loc loc1 loc2 = Loc.merge loc1 loc2 = loc2 in
let best_loc =
(* trace is with innermost call coming first *)
let rec aux best_loc = function