-
Notifications
You must be signed in to change notification settings - Fork 167
Commit
This commit does not belong to any branch on this repository, and may belong to a fork outside of the repository.
Merge pull request #1281 from affeldt-aist/mathcomp-1.11.0
mathcomp: release 1.11.0
- Loading branch information
Showing
6 changed files
with
156 additions
and
0 deletions.
There are no files selected for viewing
27 changes: 27 additions & 0 deletions
27
released/packages/coq-mathcomp-algebra/coq-mathcomp-algebra.1.11.0/opam
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1,27 @@ | ||
opam-version: "2.0" | ||
maintainer: "Mathematical Components <[email protected]>" | ||
|
||
homepage: "https://math-comp.github.io/" | ||
bug-reports: "https://github.com/math-comp/math-comp/issues" | ||
dev-repo: "git+https://github.com/math-comp/math-comp.git" | ||
license: "CECILL-B" | ||
|
||
build: [ make "-C" "mathcomp/algebra" "-j" "%{jobs}%" ] | ||
install: [ make "-C" "mathcomp/algebra" "install" ] | ||
depends: [ "coq-mathcomp-fingroup" { = version } ] | ||
|
||
tags: [ "keyword:algebra" "keyword:small scale reflection" "keyword:mathematical components" "keyword:odd order theorem" "logpath:mathcomp.algebra" ] | ||
authors: [ "Jeremy Avigad <>" "Andrea Asperti <>" "Stephane Le Roux <>" "Yves Bertot <>" "Laurence Rideau <>" "Enrico Tassi <>" "Ioana Pasca <>" "Georges Gonthier <>" "Sidi Ould Biha <>" "Cyril Cohen <>" "Francois Garillot <>" "Alexey Solovyev <>" "Russell O'Connor <>" "Laurent Théry <>" "Assia Mahboubi <>" ] | ||
|
||
synopsis: "Mathematical Components Library on Algebra" | ||
description: """ | ||
This library contains definitions and theorems about discrete | ||
(i.e. with decidable equality) algebraic structures : ring, fields, | ||
ordered fields, real fields, modules, algebras, integers, rational | ||
numbers, polynomials, matrices, vector spaces... | ||
""" | ||
|
||
url { | ||
src: "https://github.com/math-comp/math-comp/archive/mathcomp-1.11.0.tar.gz" | ||
checksum: "sha256=b16108320f77d15dd19ecc5aad90775b576edfa50c971682a1a439f6d364fef6" | ||
} |
25 changes: 25 additions & 0 deletions
25
released/packages/coq-mathcomp-character/coq-mathcomp-character.1.11.0/opam
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1,25 @@ | ||
opam-version: "2.0" | ||
maintainer: "Mathematical Components <[email protected]>" | ||
|
||
homepage: "https://math-comp.github.io/" | ||
bug-reports: "https://github.com/math-comp/math-comp/issues" | ||
dev-repo: "git+https://github.com/math-comp/math-comp.git" | ||
license: "CECILL-B" | ||
|
||
build: [ make "-C" "mathcomp/character" "-j" "%{jobs}%" ] | ||
install: [ make "-C" "mathcomp/character" "install" ] | ||
depends: [ "coq-mathcomp-field" { = version } ] | ||
|
||
tags: [ "keyword:algebra" "keyword:character" "keyword:small scale reflection" "keyword:mathematical components" "keyword:odd order theorem" "logpath:mathcomp.character" ] | ||
authors: [ "Jeremy Avigad <>" "Andrea Asperti <>" "Stephane Le Roux <>" "Yves Bertot <>" "Laurence Rideau <>" "Enrico Tassi <>" "Ioana Pasca <>" "Georges Gonthier <>" "Sidi Ould Biha <>" "Cyril Cohen <>" "Francois Garillot <>" "Alexey Solovyev <>" "Russell O'Connor <>" "Laurent Théry <>" "Assia Mahboubi <>" ] | ||
|
||
synopsis: "Mathematical Components Library on character theory" | ||
description:""" | ||
This library contains definitions and theorems about group | ||
representations, characters and class functions. | ||
""" | ||
|
||
url { | ||
src: "https://github.com/math-comp/math-comp/archive/mathcomp-1.11.0.tar.gz" | ||
checksum: "sha256=b16108320f77d15dd19ecc5aad90775b576edfa50c971682a1a439f6d364fef6" | ||
} |
25 changes: 25 additions & 0 deletions
25
released/packages/coq-mathcomp-field/coq-mathcomp-field.1.11.0/opam
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1,25 @@ | ||
opam-version: "2.0" | ||
maintainer: "Mathematical Components <[email protected]>" | ||
|
||
homepage: "https://math-comp.github.io/" | ||
bug-reports: "https://github.com/math-comp/math-comp/issues" | ||
dev-repo: "git+https://github.com/math-comp/math-comp.git" | ||
license: "CECILL-B" | ||
|
||
build: [ make "-C" "mathcomp/field" "-j" "%{jobs}%" ] | ||
install: [ make "-C" "mathcomp/field" "install" ] | ||
depends: [ "coq-mathcomp-solvable" { = version } ] | ||
|
||
tags: [ "keyword:algebra" "keyword:field" "keyword:small scale reflection" "keyword:mathematical components" "keyword:odd order theorem" "logpath:mathcomp.field" ] | ||
authors: [ "Jeremy Avigad <>" "Andrea Asperti <>" "Stephane Le Roux <>" "Yves Bertot <>" "Laurence Rideau <>" "Enrico Tassi <>" "Ioana Pasca <>" "Georges Gonthier <>" "Sidi Ould Biha <>" "Cyril Cohen <>" "Francois Garillot <>" "Alexey Solovyev <>" "Russell O'Connor <>" "Laurent Théry <>" "Assia Mahboubi <>" ] | ||
|
||
synopsis: "Mathematical Components Library on Fields" | ||
description:""" | ||
This library contains definitions and theorems about field extensions, | ||
galois theory, algebraic numbers, cyclotomic polynomials... | ||
""" | ||
|
||
url { | ||
src: "https://github.com/math-comp/math-comp/archive/mathcomp-1.11.0.tar.gz" | ||
checksum: "sha256=b16108320f77d15dd19ecc5aad90775b576edfa50c971682a1a439f6d364fef6" | ||
} |
25 changes: 25 additions & 0 deletions
25
released/packages/coq-mathcomp-fingroup/coq-mathcomp-fingroup.1.11.0/opam
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1,25 @@ | ||
opam-version: "2.0" | ||
maintainer: "Mathematical Components <[email protected]>" | ||
|
||
homepage: "https://math-comp.github.io/" | ||
bug-reports: "https://github.com/math-comp/math-comp/issues" | ||
dev-repo: "git+https://github.com/math-comp/math-comp.git" | ||
license: "CECILL-B" | ||
|
||
build: [ make "-C" "mathcomp/fingroup" "-j" "%{jobs}%" ] | ||
install: [ make "-C" "mathcomp/fingroup" "install" ] | ||
depends: [ "coq-mathcomp-ssreflect" { = version } ] | ||
|
||
tags: [ "keyword:finite groups" "keyword:small scale reflection" "keyword:mathematical components" "keyword:odd order theorem" "logpath:mathcomp.fingroup" ] | ||
authors: [ "Jeremy Avigad <>" "Andrea Asperti <>" "Stephane Le Roux <>" "Yves Bertot <>" "Laurence Rideau <>" "Enrico Tassi <>" "Ioana Pasca <>" "Georges Gonthier <>" "Sidi Ould Biha <>" "Cyril Cohen <>" "Francois Garillot <>" "Alexey Solovyev <>" "Russell O'Connor <>" "Laurent Théry <>" "Assia Mahboubi <>" ] | ||
|
||
synopsis: "Mathematical Components Library on finite groups" | ||
description: """ | ||
This library contains definitions and theorems about finite groups, | ||
group quotients, group morphisms, group presentation, group action... | ||
""" | ||
|
||
url { | ||
src: "https://github.com/math-comp/math-comp/archive/mathcomp-1.11.0.tar.gz" | ||
checksum: "sha256=b16108320f77d15dd19ecc5aad90775b576edfa50c971682a1a439f6d364fef6" | ||
} |
25 changes: 25 additions & 0 deletions
25
released/packages/coq-mathcomp-solvable/coq-mathcomp-solvable.1.11.0/opam
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1,25 @@ | ||
opam-version: "2.0" | ||
maintainer: "Mathematical Components <[email protected]>" | ||
|
||
homepage: "https://math-comp.github.io/" | ||
bug-reports: "https://github.com/math-comp/math-comp/issues" | ||
dev-repo: "git+https://github.com/math-comp/math-comp.git" | ||
license: "CECILL-B" | ||
|
||
build: [ make "-C" "mathcomp/solvable" "-j" "%{jobs}%" ] | ||
install: [ make "-C" "mathcomp/solvable" "install" ] | ||
depends: [ "coq-mathcomp-algebra" { = version } ] | ||
|
||
tags: [ "keyword:finite groups" "keyword:Feit Thompson theorem" "keyword:small scale reflection" "keyword:mathematical components" "keyword:odd order theorem" "logpath:mathcomp.solvable" ] | ||
authors: [ "Jeremy Avigad <>" "Andrea Asperti <>" "Stephane Le Roux <>" "Yves Bertot <>" "Laurence Rideau <>" "Enrico Tassi <>" "Ioana Pasca <>" "Georges Gonthier <>" "Sidi Ould Biha <>" "Cyril Cohen <>" "Francois Garillot <>" "Alexey Solovyev <>" "Russell O'Connor <>" "Laurent Théry <>" "Assia Mahboubi <>" ] | ||
|
||
synopsis: "Mathematical Components Library on finite groups (II)" | ||
|
||
description:""" | ||
This library contains more definitions and theorems about finite groups. | ||
""" | ||
|
||
url { | ||
src: "https://github.com/math-comp/math-comp/archive/mathcomp-1.11.0.tar.gz" | ||
checksum: "sha256=b16108320f77d15dd19ecc5aad90775b576edfa50c971682a1a439f6d364fef6" | ||
} |
29 changes: 29 additions & 0 deletions
29
released/packages/coq-mathcomp-ssreflect/coq-mathcomp-ssreflect.1.11.0/opam
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1,29 @@ | ||
opam-version: "2.0" | ||
maintainer: "Mathematical Components <[email protected]>" | ||
|
||
homepage: "https://math-comp.github.io/" | ||
bug-reports: "https://github.com/math-comp/math-comp/issues" | ||
dev-repo: "git+https://github.com/math-comp/math-comp.git" | ||
license: "CECILL-B" | ||
|
||
build: [ make "-C" "mathcomp/ssreflect" "-j" "%{jobs}%" ] | ||
install: [ make "-C" "mathcomp/ssreflect" "install" ] | ||
depends: [ "coq" { ((>= "8.7" & < "8.13~") )} ] | ||
|
||
tags: [ "keyword:small scale reflection" "keyword:mathematical components" "keyword:odd order theorem" "logpath:mathcomp.ssreflect" ] | ||
authors: [ "Jeremy Avigad <>" "Andrea Asperti <>" "Stephane Le Roux <>" "Yves Bertot <>" "Laurence Rideau <>" "Enrico Tassi <>" "Ioana Pasca <>" "Georges Gonthier <>" "Sidi Ould Biha <>" "Cyril Cohen <>" "Francois Garillot <>" "Alexey Solovyev <>" "Russell O'Connor <>" "Laurent Théry <>" "Assia Mahboubi <>" ] | ||
|
||
synopsis: "Small Scale Reflection" | ||
description: """ | ||
This library includes the small scale reflection proof language | ||
extension and the minimal set of libraries to take advantage of it. | ||
This includes libraries on lists (seq), boolean and boolean | ||
predicates, natural numbers and types with decidable equality, | ||
finite types, finite sets, finite functions, finite graphs, basic arithmetics | ||
and prime numbers, big operators | ||
""" | ||
|
||
url { | ||
src: "https://github.com/math-comp/math-comp/archive/mathcomp-1.11.0.tar.gz" | ||
checksum: "sha256=b16108320f77d15dd19ecc5aad90775b576edfa50c971682a1a439f6d364fef6" | ||
} |