Skip to content

Commit

Permalink
Merge pull request #2684 from palmskog/graph-theory-0.9.3
Browse files Browse the repository at this point in the history
add graph theory 0.9.3
  • Loading branch information
palmskog authored Aug 21, 2023
2 parents 78f56fa + 435fc0a commit 25ddca6
Show file tree
Hide file tree
Showing 2 changed files with 81 additions and 0 deletions.
Original file line number Diff line number Diff line change
@@ -0,0 +1,39 @@
opam-version: "2.0"
maintainer: "[email protected]"

homepage: "https://github.com/coq-community/graph-theory"
dev-repo: "git+https://github.com/coq-community/graph-theory.git"
bug-reports: "https://github.com/coq-community/graph-theory/issues"
license: "CECILL-B"

synopsis: "Graph theory results on planarity in Coq and MathComp"
description: """
Formal definitions and results on graph planarity in Coq using the Mathematical Components
library, including Wagner's Theorem. Relies on hypermaps and other notions developed
as part of the Coq proof of the Four-Color Theorem."""

build: ["dune" "build" "-p" name "-j" jobs]
depends: [
"dune" {>= "2.8"}
"coq" {>= "8.16" & < "8.19"}
"coq-mathcomp-ssreflect" {>= "2.0"}
"coq-graph-theory" {= version}
"coq-fourcolor"
]

tags: [
"category:Computer Science/Graph Theory"
"keyword:graph theory"
"keyword:planarity"
"logpath:GraphTheory.planar"
"date:2023-08-21"
]
authors: [
"Christian Doczkal"
"Damien Pous"
]

url {
src: "https://github.com/coq-community/graph-theory/archive/v0.9.3.tar.gz"
checksum: "sha512=1cc5fef0c862d8a52ebf63dad547a996b57b61d2e13ec06245ba37fee1deaccd9cf9b90ad965c6c93a06d7c197810cdabb78bf2f85f803e1f8133bf93e51dc73"
}
42 changes: 42 additions & 0 deletions released/packages/coq-graph-theory/coq-graph-theory.0.9.3/opam
Original file line number Diff line number Diff line change
@@ -0,0 +1,42 @@
opam-version: "2.0"
maintainer: "[email protected]"

homepage: "https://github.com/coq-community/graph-theory"
dev-repo: "git+https://github.com/coq-community/graph-theory.git"
bug-reports: "https://github.com/coq-community/graph-theory/issues"
license: "CECILL-B"

synopsis: "General graph theory definitions and results in Coq and MathComp"
description: """
Formalized general graph theory definitions and results using Coq and
the Mathematical Components library, including various standard results
from the literature (e.g., Menger's Theorem and Hall's Marriage Theorem)."""

build: ["dune" "build" "-p" name "-j" jobs]
depends: [
"dune" {>= "2.8"}
"coq" {>= "8.16" & < "8.19"}
"coq-mathcomp-ssreflect" {>= "2.0"}
"coq-mathcomp-algebra"
"coq-mathcomp-finmap"
"coq-hierarchy-builder" {>= "1.4.0"}
]

tags: [
"category:Computer Science/Graph Theory"
"keyword:graph theory"
"keyword:minors"
"keyword:treewidth"
"keyword:algebra"
"logpath:GraphTheory.core"
"date:2023-08-21"
]
authors: [
"Christian Doczkal"
"Damien Pous"
]

url {
src: "https://github.com/coq-community/graph-theory/archive/v0.9.3.tar.gz"
checksum: "sha512=1cc5fef0c862d8a52ebf63dad547a996b57b61d2e13ec06245ba37fee1deaccd9cf9b90ad965c6c93a06d7c197810cdabb78bf2f85f803e1f8133bf93e51dc73"
}

0 comments on commit 25ddca6

Please sign in to comment.