aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4191.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-04-21 15:54:26 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-04-21 15:56:56 +0200
commit7d261ef454e918c70b8fff1dd10bbe0fbdcb57a8 (patch)
tree385ed91f0215e4411d02ad81c932976758f830a0 /test-suite/bugs/closed/4191.v
parentce6bbd05b7d741750228956a7e045cb202ec0e74 (diff)
Fixing #3376 and #4191 (wrong index of maximally-inserted implicit argument
in the presence of let-ins).
Diffstat (limited to 'test-suite/bugs/closed/4191.v')
-rw-r--r--test-suite/bugs/closed/4191.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4191.v b/test-suite/bugs/closed/4191.v
new file mode 100644
index 000000000..290bb384d
--- /dev/null
+++ b/test-suite/bugs/closed/4191.v
@@ -0,0 +1,5 @@
+(* Test maximal implicit arguments in the presence of let-ins *)
+Definition foo (x := 1) {y : nat} (H : y = y) : True := I.
+Definition bar {y : nat} (x := 1) (H : y = y) : True := I.
+Check bar (eq_refl 1).
+Check foo (eq_refl 1).