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 /test-suite | |
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
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/bugs/closed/shouldsucceed/1905.v | 2 | ||||
-rw-r--r-- | test-suite/bugs/closed/shouldsucceed/1939.v | 2 |
2 files changed, 2 insertions, 2 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. |