aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3210.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-02-27 14:24:19 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-02-27 16:59:29 +0100
commit172388eab4f34da71d82c4fab269bd6426c73853 (patch)
treed92e642bdcbb9f805c61ca7a7652b1cc9205a86d /test-suite/bugs/closed/3210.v
parent1388171a48d8e068d5d0ed93b74faa4ac7da5f7f (diff)
Fixing first part of bug #3210 (inference of pattern-matching return
clause in the presence of let-ins in the arity of inductive type).
Diffstat (limited to 'test-suite/bugs/closed/3210.v')
-rw-r--r--test-suite/bugs/closed/3210.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3210.v b/test-suite/bugs/closed/3210.v
new file mode 100644
index 000000000..e66bf922d
--- /dev/null
+++ b/test-suite/bugs/closed/3210.v
@@ -0,0 +1,9 @@
+(* Test support of let-in in arity of inductive types *)
+
+Inductive Foo : let X := Set in X :=
+| I : Foo.
+
+Definition foo (x : Foo) : bool :=
+ match x with
+ I => true
+ end.