aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/5205.v
diff options
context:
space:
mode:
authorGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2017-06-08 14:54:39 +0200
committerGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2017-06-08 14:56:07 +0200
commit09cbae6c995c3e94ac8f0e53e6857da8e491a2fe (patch)
tree63834ae420a97b7583177df9521f57b01d5d0d82 /test-suite/bugs/closed/5205.v
parentce1e1dba837ad6e2c79ff7e531b5e3adea3cd327 (diff)
Adding a test case as requested in bug 5205.
Diffstat (limited to 'test-suite/bugs/closed/5205.v')
-rw-r--r--test-suite/bugs/closed/5205.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5205.v b/test-suite/bugs/closed/5205.v
new file mode 100644
index 000000000..406f37a4b
--- /dev/null
+++ b/test-suite/bugs/closed/5205.v
@@ -0,0 +1,6 @@
+Definition foo (n : nat) (m : nat) : nat := m.
+
+Arguments foo {_} _, _ _.
+
+Check foo 1 1.
+Check foo (n:=1) 1.