aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/unification.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-20 07:08:45 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-20 07:08:45 +0000
commit6d72bed68ae739c3c513cd50fcbadf92e576f6da (patch)
tree3fb2e952e2171d6e5705ff9b58050cd533371e81 /test-suite/success/unification.v
parent8dd3376e5d7179b8185ba55be1e66b19e65deaec (diff)
Retrait d'un test commité par erreur en 10947
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10949 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/unification.v')
-rw-r--r--test-suite/success/unification.v8
1 files changed, 0 insertions, 8 deletions
diff --git a/test-suite/success/unification.v b/test-suite/success/unification.v
index 3d935cd1d..91ee18ea4 100644
--- a/test-suite/success/unification.v
+++ b/test-suite/success/unification.v
@@ -126,11 +126,3 @@ intros.
exists (fun n => match n with O => a | S n' => f' n' end).
constructor.
Qed.
-
-(* Why this not work, even, without the "fix" to #1851 *)
-
-Goal forall X (a:X 0) (f':forall n:nat, X n), (exists f : forall n:nat, X n, True).
-intros.
-exists (fun n => match n with O => a | S n' => f' n' end).
-constructor.
-Qed.