aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-01-31 07:43:40 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-01-31 07:43:40 +0100
commit5b264fba25a996bc14c2b6dc47bc24e16fb444c7 (patch)
tree84c4058ca31758153e943cc2bdffde9184b94401 /test-suite
parent89dbc7ded0852258ef205263bfe618600168c52c (diff)
parent7321b745ab873e311a421fff0b791faa6a89580b (diff)
Merge PR #6656: Fix #5747: "make validate" fails with "bad recursive trees"
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/coqchk/include.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/coqchk/include.v b/test-suite/coqchk/include.v
new file mode 100644
index 000000000..6232c1b80
--- /dev/null
+++ b/test-suite/coqchk/include.v
@@ -0,0 +1,11 @@
+(* See https://github.com/coq/coq/issues/5747 *)
+Module Type S.
+End S.
+
+Module N.
+Inductive I := .
+End N.
+
+Module M : S.
+ Include N.
+End M.