aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/3946.v
diff options
context:
space:
mode:
authorGravatar Xavier Clerc <xavier.clerc@inria.fr>2015-01-28 14:26:19 +0100
committerGravatar Xavier Clerc <xavier.clerc@inria.fr>2015-01-28 14:26:19 +0100
commit51b15993cb4a9cc2521b6107b7f4195b21040087 (patch)
tree88770fda6bf2cac9ecee156f9869f9974a0bf2dd /test-suite/bugs/opened/3946.v
parent754e66eb2878eb964e0369226ae809ecadb1b376 (diff)
Several reproduction cases for the test suite.
Diffstat (limited to 'test-suite/bugs/opened/3946.v')
-rw-r--r--test-suite/bugs/opened/3946.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/bugs/opened/3946.v b/test-suite/bugs/opened/3946.v
new file mode 100644
index 000000000..e77bdbc65
--- /dev/null
+++ b/test-suite/bugs/opened/3946.v
@@ -0,0 +1,11 @@
+Require Import ZArith.
+
+Inductive foo := Foo : Z.le 0 1 -> foo.
+
+Definition bar (f : foo) := let (f) := f in f.
+
+(* Doesn't work: *)
+(* Arguments bar f.*)
+
+(* Does work *)
+Arguments bar f _.