aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/auto.ml
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-10-04 14:50:45 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-10-06 10:01:19 +0200
commit07f4e6b07775052cc1c5dc34cdfa7ad4eacfa94f (patch)
tree4bb7a90d8474b038434b732fb24b9b9d69e937c3 /tactics/auto.ml
parentefce61af32ff1b09a21dcf88bca7d6609a0bfd27 (diff)
Fix bug #4354: interpret hints in the right env and sigma.
Diffstat (limited to 'tactics/auto.ml')
-rw-r--r--tactics/auto.ml7
1 files changed, 5 insertions, 2 deletions
diff --git a/tactics/auto.ml b/tactics/auto.ml
index 72ba9e0bd..e5fdf6a7c 100644
--- a/tactics/auto.ml
+++ b/tactics/auto.ml
@@ -309,7 +309,8 @@ let rec trivial_fail_db dbg mod_delta db_list local_db =
let decl = Tacmach.New.pf_last_hyp (Proofview.Goal.assume gl) in
let hyp = Context.map_named_declaration nf decl in
let hintl = make_resolve_hyp env sigma hyp
- in trivial_fail_db dbg mod_delta db_list (Hint_db.add_list hintl local_db)
+ in trivial_fail_db dbg mod_delta db_list
+ (Hint_db.add_list env sigma hintl local_db)
end)
in
Proofview.Goal.enter begin fun gl ->
@@ -438,7 +439,9 @@ let possible_resolve dbg mod_delta db_list local_db cl =
with Not_found -> []
let extend_local_db decl db gl =
- Hint_db.add_list (make_resolve_hyp (Tacmach.New.pf_env gl) (Proofview.Goal.sigma gl) decl) db
+ let env = Tacmach.New.pf_env gl in
+ let sigma = Proofview.Goal.sigma gl in
+ Hint_db.add_list env sigma (make_resolve_hyp env sigma decl) db
(* Introduce an hypothesis, then call the continuation tactic [kont]
with the hint db extended with the so-obtained hypothesis *)