aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-10-15 16:27:37 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-10-15 16:28:34 +0200
commitc3b9a7bf9fcd162628ce6a2a544652ca096cfe54 (patch)
tree28459c0899c47ee8f2229c602cab3d1637985f68 /test-suite
parent7c047370dc9032e3ded3365a45de5b92e7c9033f (diff)
Fix bug #5145: Anomaly: index to an anonymous variable.
When printing evar constraints, we ensure that every variable from the rel context has a name.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/5145.v10
1 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5145.v b/test-suite/bugs/closed/5145.v
new file mode 100644
index 000000000..0533d21e0
--- /dev/null
+++ b/test-suite/bugs/closed/5145.v
@@ -0,0 +1,10 @@
+Class instructions :=
+ {
+ W : Type;
+ ldi : nat -> W
+ }.
+
+Fail Definition foo :=
+ let y2 := ldi 0 in
+ let '(CF, _) := (true, 0) in
+ y2.