diff options
author | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2009-04-20 15:28:16 +0000 |
---|---|---|
committer | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2009-04-20 15:28:16 +0000 |
commit | 70b225dce6fa0e2bf4763f1669f1ed9705d77c11 (patch) | |
tree | da5ad57bdd3758cb3f5fa34cd5128b0bd19e46a0 | |
parent | 4aa97e1314fdeedd4e1e5a1574671057d889f659 (diff) |
Fix wrong pattern in Morphisms. Fix bug scripts to reflect the fact that
Setoid doesn't export Program.Basics anymore.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12095 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r-- | test-suite/bugs/closed/shouldsucceed/1905.v | 2 | ||||
-rw-r--r-- | test-suite/bugs/closed/shouldsucceed/1939.v | 2 | ||||
-rw-r--r-- | theories/Classes/Morphisms.v | 4 |
3 files changed, 4 insertions, 4 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/1905.v b/test-suite/bugs/closed/shouldsucceed/1905.v index bd7fd7967..fb2725c97 100644 --- a/test-suite/bugs/closed/shouldsucceed/1905.v +++ b/test-suite/bugs/closed/shouldsucceed/1905.v @@ -1,5 +1,5 @@ -Require Import Setoid. +Require Import Setoid Program. Axiom t : Set. Axiom In : nat -> t -> Prop. diff --git a/test-suite/bugs/closed/shouldsucceed/1939.v b/test-suite/bugs/closed/shouldsucceed/1939.v index 0399b1124..3aa55e834 100644 --- a/test-suite/bugs/closed/shouldsucceed/1939.v +++ b/test-suite/bugs/closed/shouldsucceed/1939.v @@ -1,4 +1,4 @@ -Require Import Setoid. +Require Import Setoid Program.Basics. Parameter P : nat -> Prop. Parameter R : nat -> nat -> Prop. diff --git a/theories/Classes/Morphisms.v b/theories/Classes/Morphisms.v index d2bc277e9..e2ab8b118 100644 --- a/theories/Classes/Morphisms.v +++ b/theories/Classes/Morphisms.v @@ -424,8 +424,8 @@ Proof. firstorder. Qed. Lemma inverse2 `(subrelation A R R') : subrelation R (inverse (inverse R')). Proof. firstorder. Qed. -Hint Extern 1 (subrelation (flip (flip _)) _) => eapply @inverse1 : typeclass_instances. -Hint Extern 1 (subrelation _ (flip (flip _))) => eapply @inverse2 : typeclass_instances. +Hint Extern 1 (subrelation (flip _) _) => eapply @inverse1 : typeclass_instances. +Hint Extern 1 (subrelation _ (flip _)) => eapply @inverse2 : typeclass_instances. (** Once we have normalized, we will apply this instance to simplify the problem. *) |