Skip to content

Commit

Permalink
Add odoc warnings for empty packages.
Browse files Browse the repository at this point in the history
From an OCaml library point of view.
  • Loading branch information
Zimmi48 committed Apr 6, 2021
1 parent 56c32d8 commit acae2dc
Show file tree
Hide file tree
Showing 8 changed files with 26 additions and 0 deletions.
3 changes: 3 additions & 0 deletions doc/dune
Expand Up @@ -63,3 +63,6 @@
(files (refman-html as html/refman) (refman-pdf as pdf/refman))
(section doc)
(package coq-doc))

(documentation
(package coq-doc))
3 changes: 3 additions & 0 deletions doc/index.mld
@@ -0,0 +1,3 @@
{0 coq-doc }

The coq-doc package only contains user documentation on the Coq proof assistant and no OCaml library.
3 changes: 3 additions & 0 deletions dune
Expand Up @@ -35,3 +35,6 @@
(deps test-suite/summary.log))

; (dirs (:standard _build_ci))

(documentation
(package coq))
3 changes: 3 additions & 0 deletions ide/coqide/dune
Expand Up @@ -51,6 +51,9 @@
(modes exe byte)
(libraries coqide_gui))

(documentation
(package coqide))

; Input-method bindings
(executable
(name default_bindings_src)
Expand Down
3 changes: 3 additions & 0 deletions ide/coqide/index.mld
@@ -0,0 +1,3 @@
{0 coqide }

The coqide package only contains the CoqIDE executable and no OCaml library.
5 changes: 5 additions & 0 deletions index.mld
@@ -0,0 +1,5 @@
{0 coq }

The coq package is a virtual package gathering the coq-core and coq-stdlib packages.

For the documentation of the OCaml API of Coq, see the coq-core package.
3 changes: 3 additions & 0 deletions theories/dune
Expand Up @@ -34,3 +34,6 @@
coq-core.plugins.derive))

(include_subdirs qualified)

(documentation
(package coq-stdlib))
3 changes: 3 additions & 0 deletions theories/index.mld
@@ -0,0 +1,3 @@
{0 coq-stdlib }

The coq-stdlib package only contains Coq theory files for the standard library and no OCaml libraries.

0 comments on commit acae2dc

Please sign in to comment.