Skip to content

Commit

Permalink
Backport from opam repo
Browse files Browse the repository at this point in the history
C.f. coq/opam#3293

(cherry picked from commit 4495ca0)
  • Loading branch information
proux01 authored and ppedrot committed Jan 20, 2025
1 parent b83bd97 commit ef14755
Show file tree
Hide file tree
Showing 3 changed files with 35 additions and 1 deletion.
14 changes: 14 additions & 0 deletions coq-core.opam
Original file line number Diff line number Diff line change
Expand Up @@ -2,6 +2,20 @@
opam-version: "2.0"
version: "dev"
synopsis: "Compatibility binaries for Coq after the Rocq renaming"
description: """
The Rocq Prover is an interactive theorem prover, or proof assistant. 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 compatibility binaries to call Rocq
through previous Coq commands like coqc coqtop,..."""
maintainer: ["The Rocq development team <[email protected]>"]
authors: ["The Rocq development team, INRIA, CNRS, and contributors"]
license: "LGPL-2.1-only"
Expand Down
18 changes: 17 additions & 1 deletion dune-project
Original file line number Diff line number Diff line change
Expand Up @@ -30,6 +30,9 @@
(ocamlfind (>= 1.8.1))
(zarith (>= 1.11))
(conf-linux-libc-dev (= :os "linux")))
(conflicts
(coq (< 8.17))
(coq-core (< 8.21)))
(depopts rocq-native memprof-limits memtrace)
(synopsis "The Rocq Prover -- Core Binaries and Tools")
(description "The Rocq Prover is an interactive theorem prover, or proof assistant. It provides
Expand All @@ -54,7 +57,20 @@ prelude, now living in the rocq-core package."))
(name coq-core)
(depends
(rocq-runtime (= :version)))
(synopsis "Compatibility binaries for Coq after the Rocq renaming"))
(synopsis "Compatibility binaries for Coq after the Rocq renaming")
(description "The Rocq Prover is an interactive theorem prover, or proof assistant. 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 compatibility binaries to call Rocq
through previous Coq commands like coqc coqtop,..."))

(package
(name rocq-core)
Expand Down
4 changes: 4 additions & 0 deletions rocq-runtime.opam
Original file line number Diff line number Diff line change
Expand Up @@ -35,6 +35,10 @@ depends: [
"odoc" {with-doc}
]
depopts: ["rocq-native" "memprof-limits" "memtrace"]
conflicts: [
"coq" {< "8.17"}
"coq-core" {< "8.21"}
]
dev-repo: "git+https://github.com/coq/coq.git"
build: [
["dune" "subst"] {dev}
Expand Down

0 comments on commit ef14755

Please sign in to comment.