DEBSOURCES
Skip Quicknav
sources / coq-doc / 8.16.1-1 / test-suite / coqchk / include.v
1234567891011
(* 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.