aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-01-25 00:18:28 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-01-25 00:18:28 +0100
commit9273e81b853a8e107da57e902ce130ad1e54f928 (patch)
tree3cc7c657243f94d90ed9f3205492a222dc733ee2 /test-suite
parent6638997f6c975e88a35ccd260d0c40c287391a45 (diff)
Adding a test for bug #3023.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/3023.v8
1 files changed, 5 insertions, 3 deletions
diff --git a/test-suite/bugs/closed/3023.v b/test-suite/bugs/closed/3023.v
index ed4895115..70a1491e1 100644
--- a/test-suite/bugs/closed/3023.v
+++ b/test-suite/bugs/closed/3023.v
@@ -1,5 +1,3 @@
-(* Checking use of eta on Flexible/Rigid and SemiFlexible/Rigid unif problems *)
-
Set Implicit Arguments.
Generalizable All Variables.
@@ -14,6 +12,7 @@ Record Category {obj : Type} :=
Section DiscreteAdjoints.
+
Let C := {|
Morphism := (fun X Y : Type => X -> Y);
Identity := (fun X : Type => (fun x : X => x));
@@ -28,4 +27,7 @@ Section DiscreteAdjoints.
revert ObjectFunctor.
intro ObjectFunctor.
simpl in ObjectFunctor.
- revert ObjectFunctor. (* Used to failed in 8.4 up to 16 April 2013 *)
+ revert ObjectFunctor.
+ Abort.
+
+End DiscreteAdjoints.