Skip to content

Commit

Permalink
math-comp-school-2022
Browse files Browse the repository at this point in the history
  • Loading branch information
gares committed Nov 17, 2022
1 parent bb768b8 commit 86c307c
Show file tree
Hide file tree
Showing 11 changed files with 244 additions and 105 deletions.
10 changes: 3 additions & 7 deletions .github/workflows/macos.yml
Original file line number Diff line number Diff line change
Expand Up @@ -12,9 +12,7 @@ name: Macos
on:
push:
branches:
- 2021.02
- 2021.09
- main
- math-comp-school-2022
pull_request:
branches:
- '**'
Expand Down Expand Up @@ -48,8 +46,7 @@ jobs:
fail-fast: false
matrix:
variant:
- '8.16~2022.09~beta1'
- '8.15~2022.04'
- 'math-comp-school-2022'

steps:
- name: Git checkout
Expand Down Expand Up @@ -123,8 +120,7 @@ jobs:
fail-fast: false
matrix:
variant:
- '8.16~2022.09~beta1'
- '8.15~2022.04'
- 'math-comp-school-2022'

steps:
- name: Install bash
Expand Down
13 changes: 3 additions & 10 deletions .github/workflows/ubuntu.yml
Original file line number Diff line number Diff line change
Expand Up @@ -12,9 +12,7 @@ name: Ubuntu
on:
push:
branches:
- 2021.02
- 2021.09
- main
- math-comp-school-2022
pull_request:
branches:
- '**'
Expand All @@ -39,7 +37,7 @@ on:
env:
PLATFORM: -extent=x -parallel=p -jobs=2 -large=i -compcert=y -unimath=n -set-switch=y
COQREGTESTING: y
SNAP_PICK: 8.16~2022.09~beta1
SNAP_PICK: math-comp-school-2022

###############################################################################
# Ubuntu
Expand All @@ -57,12 +55,7 @@ jobs:
matrix:
variant:
# This should contain all picks introduced in the current release + all original picks of all Coq versions
- '8.16~2022.09~beta1'
- '8.15~2022.09~beta1'
- '8.15~2022.04'
- '8.14~2022.01'
- '8.13~2021.02'
- '8.12'
- 'math-comp-school-2022'

steps:
- name: Git checkout
Expand Down
79 changes: 0 additions & 79 deletions .github/workflows/ubuntu_dev.yml

This file was deleted.

12 changes: 3 additions & 9 deletions .github/workflows/windows.yml
Original file line number Diff line number Diff line change
Expand Up @@ -12,9 +12,7 @@ name: Windows
on:
push:
branches:
- 2021.02
- 2021.09
- main
- math-comp-school-2022
pull_request:
branches:
- '**'
Expand Down Expand Up @@ -50,12 +48,10 @@ jobs:
fail-fast: false
matrix:
architecture:
- '32'
- '64'
variant:
# Keep this in sync with the Smoke test below
- '8.16~2022.09~beta1'
- '8.15~2022.04'
- 'math-comp-school-2022'

steps:
- name: Set git to use LF
Expand Down Expand Up @@ -104,11 +100,9 @@ jobs:
fail-fast: false
matrix:
architecture:
- '32'
- '64'
variant:
- '8.16~2022.09~beta1'
- '8.15~2022.04'
- 'math-comp-school-2022'

steps:
- name: 'Download Artifact'
Expand Down
Original file line number Diff line number Diff line change
@@ -0,0 +1,26 @@
opam-version: "2.0"
version: "dev"
maintainer: "Mathematical Components <mathcomp-dev@sympa.inria.fr>"

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/zipball/hierarchy-builder"
}
Original file line number Diff line number Diff line change
@@ -0,0 +1,24 @@
opam-version: "2.0"
version: "dev"
maintainer: "Mathematical Components <mathcomp-dev@sympa.inria.fr>"

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/zipball/hierarchy-builder"
}
Original file line number Diff line number Diff line change
@@ -0,0 +1,24 @@
opam-version: "2.0"
version: "dev"
maintainer: "Mathematical Components <mathcomp-dev@sympa.inria.fr>"

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/zipball/hierarchy-builder"
}
Original file line number Diff line number Diff line change
@@ -0,0 +1,24 @@
opam-version: "2.0"
version: "dev"
maintainer: "Mathematical Components <mathcomp-dev@sympa.inria.fr>"

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/zipball/hierarchy-builder"
}
Original file line number Diff line number Diff line change
@@ -0,0 +1,24 @@
opam-version: "2.0"
version: "dev"
maintainer: "Mathematical Components <mathcomp-dev@sympa.inria.fr>"

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/zipball/hierarchy-builder"
}
Original file line number Diff line number Diff line change
@@ -0,0 +1,31 @@
opam-version: "2.0"
version: "dev"
maintainer: "Mathematical Components <mathcomp-dev@sympa.inria.fr>"

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.13" & < "8.17~") | (= "dev"))}
"coq-hierarchy-builder" { >= "1.4.0"}
]

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/zipball/hierarchy-builder"
}
Loading

0 comments on commit 86c307c

Please sign in to comment.