aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-11-13 16:33:26 +0100
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-11-13 16:33:26 +0100
commit3aeb18bf1412a27309c39713e05eca2c27706ca8 (patch)
tree5545c18780cc64076ba241feb7abefb18b7b2e3f
parent2fd497d380de998c4b22b9f7167eb4023e4cd576 (diff)
Continue fix of PMP, handling setoid_rewrite in let-bound hyps correctly.
-rw-r--r--tactics/rewrite.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/tactics/rewrite.ml b/tactics/rewrite.ml
index af6953bf8..182c232ae 100644
--- a/tactics/rewrite.ml
+++ b/tactics/rewrite.ml
@@ -1505,7 +1505,7 @@ let assert_replacing id newt tac =
let after, before = List.split_when (fun (n, b, t) -> Id.equal n id) ctx in
let nc = match before with
| [] -> assert false
- | (id, b, _) :: rem -> insert_dependent env (id, b, newt) [] after @ rem
+ | (id, b, _) :: rem -> insert_dependent env (id, None, newt) [] after @ rem
in
let env' = Environ.reset_with_named_context (val_of_named_context nc) env in
Proofview.Refine.refine ~unsafe:false begin fun sigma ->