aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2018-02-13 11:15:16 +0100
committerGravatar Matthieu Sozeau <mattam@mattam.org>2018-02-19 10:24:31 +0100
commitee31c1d24e0c493bb777a58d871f5085222fbc4d (patch)
treedabeee25a553981f388b860eec2b11724db37003 /test-suite
parent4f65dfb13d8bb395abf4aa405cae9ed529302a06 (diff)
Fix #6529: nf_evar_info and check the env evars' not just the concl
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/6529.v16
1 files changed, 16 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/6529.v b/test-suite/bugs/closed/6529.v
new file mode 100644
index 000000000..8d9081999
--- /dev/null
+++ b/test-suite/bugs/closed/6529.v
@@ -0,0 +1,16 @@
+Require Import Vector Program.
+
+Program Definition append_nil_def :=
+ forall A n (ls: t A n), append ls (nil A) = ls. (* Works *)
+
+Lemma append_nil : append_nil_def. (* Works *)
+Proof.
+Admitted.
+
+Program Lemma append_nil' :
+ forall A n (ls: t A n), append ls (nil A) = ls.
+Abort.
+
+Fail Program Lemma append_nil'' :
+ forall A B n (ls: t A n), append ls (nil A) = ls.
+(* Error: Anomaly "Evar ?X25 was not declared." Please report at http://coq.inria.fr/bugs/. *)