Skip to content

Commit

Permalink
[coq.dev] Attempt to split the packages.
Browse files Browse the repository at this point in the history
We use the conditional setup outlined in Zulip, let's see how and if
this works.
  • Loading branch information
ejgallego committed Nov 8, 2021
1 parent 2697950 commit 1d3b23c
Show file tree
Hide file tree
Showing 3 changed files with 87 additions and 22 deletions.
43 changes: 43 additions & 0 deletions core-dev/packages/coq-core/coq-core.dev/opam
Original file line number Diff line number Diff line change
@@ -0,0 +1,43 @@
opam-version: "2.0"
maintainer: "[email protected]"
authors: "The Coq development team, INRIA, CNRS, and contributors."
homepage: "https://coq.inria.fr/"
bug-reports: "https://github.com/coq/coq/issues"
dev-repo: "git+https://github.com/coq/coq.git"
license: "LGPL-2.1-only"
synopsis: "Formal proof management system"
description: """
The Coq proof assistant provides a formal language to write
mathematical definitions, executable algorithms, and theorems, together
with an environment for semi-interactive development of machine-checked
proofs. Typical applications include the certification of properties of programming
languages (e.g., the CompCert compiler certification project and the
Bedrock verified low-level programming library), the formalization of
mathematics (e.g., the full formalization of the Feit-Thompson theorem
and homotopy type theory) and teaching.
"""

depopts: [
"coq-native"
]

depends: [
"ocaml" {>= "4.05.0"}
"ocamlfind" {build}
"dune" {>= "2.9.1"}
"conf-findutils" {build}
"zarith" {>= "1.10"}
]

build: [
[
"./configure"
"-prefix" prefix
"-native-compiler" "yes" {coq-native:installed} "no" {!coq-native:installed}
]
[ "dune" "build" "-p" name "-j" jobs ]
]

url {
src: "git+https://github.com/coq/coq.git#master"
}
41 changes: 41 additions & 0 deletions core-dev/packages/coq-stdlib/coq-stdlib.dev/opam
Original file line number Diff line number Diff line change
@@ -0,0 +1,41 @@
opam-version: "2.0"
maintainer: "[email protected]"
authors: "The Coq development team, INRIA, CNRS, and contributors."
homepage: "https://coq.inria.fr/"
bug-reports: "https://github.com/coq/coq/issues"
dev-repo: "git+https://github.com/coq/coq.git"
license: "LGPL-2.1-only"
synopsis: "Formal proof management system"
description: """
The Coq proof assistant provides a formal language to write
mathematical definitions, executable algorithms, and theorems, together
with an environment for semi-interactive development of machine-checked
proofs. Typical applications include the certification of properties of programming
languages (e.g., the CompCert compiler certification project and the
Bedrock verified low-level programming library), the formalization of
mathematics (e.g., the full formalization of the Feit-Thompson theorem
and homotopy type theory) and teaching.
"""

depopts: [
"coq-native"
]

depends: [
"ocaml" {>= "4.05.0"}
"ocamlfind" {build}
"dune" {>= "2.9.1"}
"conf-findutils" {build}
"zarith" {>= "1.10"}
"coq-core" {= version}
]

build: [
# This is akin to a configure step
[ "sed '1 a (mode native)' theories/dune" {coq-native:installed} ]
[ "dune" "build" "-p" name "-j" jobs ]
]

url {
src: "git+https://github.com/coq/coq.git#master"
}
25 changes: 3 additions & 22 deletions core-dev/packages/coq/coq.dev/opam
Original file line number Diff line number Diff line change
Expand Up @@ -20,29 +20,10 @@ and homotopy type theory) and teaching.
depopts: [
"coq-native"
]

depends: [
"ocaml" {>= "4.05.0"}
"ocamlfind" {build}
"dune" {>= "2.5.1"}
"conf-findutils" {build}
"zarith" {>= "1.10"}
]
build: [
[
"./configure"
"-configdir" "%{lib}%/coq/config"
"-prefix" prefix
"-mandir" man
"-docdir" doc
"-libdir" "%{lib}%/coq"
"-datadir" "%{share}%/coq"
"-coqide" "no"
"-native-compiler" "yes" {coq-native:installed} "no" {!coq-native:installed}
]
[make "-j%{jobs}%"]
]
install: [
[make "install"]
"coq-core" {= version}
"coq-stdlib" {= version}
]

url {
Expand Down

0 comments on commit 1d3b23c

Please sign in to comment.