aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-02-21 12:38:25 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-02-21 12:39:58 +0100
commitf1389e10e6bf15e0fe3fd120f4aa8e59579a16b4 (patch)
treedc3954a0823106e0139951b83a179969ae455bcd /test-suite/bugs/opened
parent4bb062f4a66c4ae5a1742e7d99fdc335de0d57a9 (diff)
Removed tests for #3900 and #3944 as open bugs.
Diffstat (limited to 'test-suite/bugs/opened')
-rw-r--r--test-suite/bugs/opened/3900.v12
-rw-r--r--test-suite/bugs/opened/3944.v4
2 files changed, 0 insertions, 16 deletions
diff --git a/test-suite/bugs/opened/3900.v b/test-suite/bugs/opened/3900.v
deleted file mode 100644
index b791b5351..000000000
--- a/test-suite/bugs/opened/3900.v
+++ /dev/null
@@ -1,12 +0,0 @@
-Global Set Primitive Projections.
-Set Implicit Arguments.
-Record sigT {A} (P : A -> Type) := existT { projT1 : A ; projT2 : P projT1 }.
-Record PreCategory := { object :> Type ; morphism : object -> object -> Type }.
-Variable A : PreCategory.
-Variable Pobj : A -> Type.
-Local Notation obj := (sigT Pobj).
-Variable Pmor : forall s d : obj, morphism A (projT1 s) (projT1 d) -> Type.
-Class Foo (x : Type) := { _ : forall y, y }.
-Local Instance ishset_pmor {s d m} : Foo (Pmor s d m).
-Proof.
- Fail SearchAbout ((forall _ _, _) -> Foo _).
diff --git a/test-suite/bugs/opened/3944.v b/test-suite/bugs/opened/3944.v
deleted file mode 100644
index 3d0deb4c5..000000000
--- a/test-suite/bugs/opened/3944.v
+++ /dev/null
@@ -1,4 +0,0 @@
-Require Import Setoid.
-Class C (T : Type) := c : T.
-Goal forall T (i : C T) (v : T), True.
-setoid_rewrite plus_n_Sm.