summaryrefslogtreecommitdiff
path: root/test-suite/coqchk/include.v
blob: 6232c1b80ff44491822f16f8e66187b2c25214b2 (plain)
1
2
3
4
5
6
7
8
9
10
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.