diff options
author | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2014-05-08 13:24:16 +0200 |
---|---|---|
committer | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2014-05-08 20:44:29 +0200 |
commit | 6522aa62d832837314dcef54735e6a4e55431571 (patch) | |
tree | f5656113b66ba2c809e80353088cf391f4243b92 /test-suite | |
parent | f87c3a55b1ad52b63ebd0af0cf9f3fb0e8e86f76 (diff) |
Simplification and improvement of "subst x" in such a way that it
works in the presence of local definitions referring to x and
dependent in other hyps or concl.
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/success/rewrite.v | 9 |
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/success/rewrite.v b/test-suite/success/rewrite.v index 08c406be9..0e1e77863 100644 --- a/test-suite/success/rewrite.v +++ b/test-suite/success/rewrite.v @@ -129,3 +129,12 @@ intros. Fail rewrite H in H0. Abort. +(* Test subst in the presence of a dependent let-in *) +(* Was not working prior to May 2014 *) + +Goal forall x y, x=y+0 -> let z := x+1 in x+1=y -> z=z -> z=x. +intros. +subst x. (* was failing *) +rewrite H0. +reflexivity. +Qed. |