Skip to content

Commit

Permalink
Merge pull request #3275 from proux01/rocq-stdlib
Browse files Browse the repository at this point in the history
[core-dev] Rename coq-stdlib -> rocq-stdlib
  • Loading branch information
ppedrot authored Jan 8, 2025
2 parents d67f549 + c1c4053 commit a17237a
Show file tree
Hide file tree
Showing 2 changed files with 54 additions and 3 deletions.
6 changes: 3 additions & 3 deletions core-dev/packages/coq-stdlib/coq-stdlib.dev/opam
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
opam-version: "2.0"
synopsis: "The Coq Proof Assistant -- Standard Library"
synopsis: "Compatibility metapackage for Coq Stdlib library after the Rocq renaming"
description: """
Coq is a formal proof management system. It provides
a formal language to write mathematical definitions, executable
Expand All @@ -22,8 +22,8 @@ doc: "https://coq.github.io/doc/"
bug-reports: "https://github.com/coq/coq/issues"
depends: [
"dune" {>= "3.8"}
"rocq-runtime"
"rocq-core" {= version}
"coq-core"
"rocq-stdlib" {= version}
"odoc" {with-doc}
]
depopts: ["coq-native"]
Expand Down
51 changes: 51 additions & 0 deletions core-dev/packages/rocq-stdlib/rocq-stdlib.dev/opam
Original file line number Diff line number Diff line change
@@ -0,0 +1,51 @@
opam-version: "2.0"
synopsis: "The Rocq Proof Assistant -- Standard Library"
description: """
Rocq is a formal proof management system. It 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, or the Bedrock verified low-level programming library), the
formalization of mathematics (e.g. the full formalization of the
Feit-Thompson theorem or homotopy type theory) and teaching.

This package includes the Rocq Standard Library, that is to say, the
set of modules usually bound to the Stdlib.* namespace."""
maintainer: ["The Rocq standard library development team"]
authors: ["The Rocq development team, INRIA, CNRS, and contributors"]
license: "LGPL-2.1-only"
homepage: "https://coq.inria.fr/"
doc: "https://coq.github.io/doc/"
bug-reports: "https://github.com/coq/coq/issues"
depends: [
"dune" {>= "3.8"}
"rocq-runtime"
"rocq-core" {= version}
"odoc" {with-doc}
]
depopts: ["coq-native"]
dev-repo: "git+https://github.com/coq/coq.git"
build: [
["sh" "-c" "echo '(dirs stdlib)' > dune"]
["dune" "subst"] {dev}
[
"stdlib/dev/with-rocq-wrap.sh"
"dune"
"build"
"-p"
name
"-j"
jobs
"@install"
"@runtest" {with-test}
"@doc" {with-doc}
]
["mv" "stdlib/rocq-stdlib.install" "."]
]

url {
src: "git+https://github.com/coq/coq.git#master"
}

0 comments on commit a17237a

Please sign in to comment.