aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/unification.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-14 21:03:43 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-14 21:03:43 +0000
commit4586e512ff1f8b7e3911959bd2ab60f465f236f9 (patch)
tree4e8ed463f055d5f40cdfc141cb60d1d4b735d2ee /test-suite/success/unification.v
parentf13aaec57df12380323edf450aec14c372422d58 (diff)
Résolution des problèmes ambigus d'inférence du type de retour des
problèmes de filtrage au nivau de consider_remaining_unif_problems (résoud en particulier le "bug" #1851). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10927 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/unification.v')
-rw-r--r--test-suite/success/unification.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/success/unification.v b/test-suite/success/unification.v
index 51b0e06e5..91ee18ea4 100644
--- a/test-suite/success/unification.v
+++ b/test-suite/success/unification.v
@@ -117,3 +117,12 @@ Inductive nonemptyT (t : Type) : Prop := nonemptyT_intro : t -> nonemptyT t.
Goal True.
try case nonemptyT_intro. (* check that it fails w/o anomaly *)
Abort.
+
+(* Test handling of return type and when it is decided to make the
+ predicate dependent or not - see "bug" #1851 *)
+
+Goal forall X (a:X) (f':nat -> X), (exists f : nat -> X, True).
+intros.
+exists (fun n => match n with O => a | S n' => f' n' end).
+constructor.
+Qed.