aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Cases-bug1834.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-10 19:36:10 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-10 19:36:10 +0000
commitcc46417aad0bb80e3617baaf37fee93f1ea3034e (patch)
tree6c890934d88f19c42467a0b8aa8114969064f399 /test-suite/success/Cases-bug1834.v
parent5d8d8e858e56c0d12cb262d5ff8e733ae7afc102 (diff)
- Amélioration nommage dans EqdepFacts suivant remarque de Arthur C.
- Test match dépendant. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11095 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/Cases-bug1834.v')
-rw-r--r--test-suite/success/Cases-bug1834.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/success/Cases-bug1834.v b/test-suite/success/Cases-bug1834.v
new file mode 100644
index 000000000..543ca0c92
--- /dev/null
+++ b/test-suite/success/Cases-bug1834.v
@@ -0,0 +1,13 @@
+(* Bug in the computation of generalization *)
+
+(* The following bug, elaborated by Bruno Barras, is solved from r11083 *)
+
+Parameter P : unit -> Prop.
+Definition T := sig P.
+Parameter Q : T -> Prop.
+Definition U := sig Q.
+Parameter a : U.
+Check (match a with exist (exist tt e2) e3 => e3=e3 end).
+
+(* There is still a form submitted by Pierre Corbineau (#1834) which fails *)
+