aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-21 16:26:38 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-21 16:26:38 +0000
commit2407beea26ae531431db3123ecba6a08acd4e3e2 (patch)
tree5e4e802879754ac32ddc3718cde22d36193b18c3 /test-suite/bugs
parent880a83169c1d1df8726d301a9f8a9fc845cc7d1e (diff)
- Correct unification for the rewrite variant of setoid_rewrite,
so that the example of bug #1425 is accepted. - Backtrack level of notations for morphism signatures to 55. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10825 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/shouldsucceed/1425.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/1425.v b/test-suite/bugs/closed/shouldsucceed/1425.v
index f5fbb8a2a..8e26209a1 100644
--- a/test-suite/bugs/closed/shouldsucceed/1425.v
+++ b/test-suite/bugs/closed/shouldsucceed/1425.v
@@ -8,6 +8,12 @@ Axiom recursion_S :
Goal forall n : nat, recursion nat 0 (fun _ _ => 1) (S n) = 1.
intro n.
+rewrite recursion_S.
+reflexivity.
+Qed.
+
+Goal forall n : nat, recursion nat 0 (fun _ _ => 1) (S n) = 1.
+intro n.
setoid_rewrite recursion_S.
reflexivity.
Qed. \ No newline at end of file