aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-10 18:28:26 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-10 18:28:26 +0000
commite121b1de13ed893a37a73c852e4e9de933eef32a (patch)
tree86522098425c086554fd70638dd622bb3cf138c1 /test-suite/bugs
parent813b9b40ce96c59f9e68b759c876a0ccbfdbf942 (diff)
- Correct handling of DependentMorphism error, using tclFAIL instead of
letting the exception go uncatched. - Reorder definitions in Morphisms, move the PER on (R ==> R') in Morphisms where it can be declared properly. Add an instance for Equivalence => Per. - Change bug#1604 test file to the new semantics of [setoid_rewrite at] - More unicode characters parsed by coqdoc. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11092 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/shouldsucceed/1604.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/1604.v b/test-suite/bugs/closed/shouldsucceed/1604.v
index 2d0991cb1..22c3df824 100644
--- a/test-suite/bugs/closed/shouldsucceed/1604.v
+++ b/test-suite/bugs/closed/shouldsucceed/1604.v
@@ -3,5 +3,5 @@ Require Import Setoid.
Parameter F : nat -> nat.
Axiom F_id : forall n : nat, n = F n.
Goal forall n : nat, F n = n.
-intro n. setoid_rewrite F_id at 2. reflexivity.
+intro n. setoid_rewrite F_id at 3. reflexivity.
Qed.