aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/auto.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-10-08 02:21:26 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-10-12 13:35:58 +0200
commit55699e2b9a91356b7d43c4096f65fb199777b9a1 (patch)
treea1b9ccff30d86f9c57794ce872fe14bbf1879575 /tactics/auto.ml
parent5539201bf25dec1b5c24634dca581e199caca4e7 (diff)
Fix bug #4958: [debug auto] should specify hint databases.
Diffstat (limited to 'tactics/auto.ml')
-rw-r--r--tactics/auto.ml11
1 files changed, 9 insertions, 2 deletions
diff --git a/tactics/auto.ml b/tactics/auto.ml
index 962af4b5c..6d1a1ae28 100644
--- a/tactics/auto.ml
+++ b/tactics/auto.ml
@@ -375,7 +375,7 @@ and my_find_search_delta db_list local_db hdc concl =
in List.map (fun x -> (Some flags,x)) l)
(local_db::db_list)
-and tac_of_hint dbg db_list local_db concl (flags, ({pat=p; code=t;poly=poly})) =
+and tac_of_hint dbg db_list local_db concl (flags, ({pat=p; code=t;poly=poly;db=dbname})) =
let tactic = function
| Res_pf (c,cl) -> unify_resolve_gen poly flags (c,cl)
| ERes_pf _ -> Proofview.V82.tactic (fun gl -> error "eres_pf")
@@ -394,7 +394,14 @@ and tac_of_hint dbg db_list local_db concl (flags, ({pat=p; code=t;poly=poly}))
| Extern tacast ->
conclPattern concl p tacast
in
- tclLOG dbg (fun () -> pr_hint t) (run_hint t tactic)
+ let pr_hint () =
+ let origin = match dbname with
+ | None -> mt ()
+ | Some n -> str " (in " ++ str n ++ str ")"
+ in
+ pr_hint t ++ origin
+ in
+ tclLOG dbg pr_hint (run_hint t tactic)
and trivial_resolve dbg mod_delta db_list local_db cl =
try