Skip to content

Commit 7ee1240

Browse files
authored
Merge pull request #3316 from yforster/coq-metacoq.1.3.4+8.20
Add packages for MetaCoq 1.3.4 on Coq 8.20
2 parents e6989c8 + 2bd8bbe commit 7ee1240

File tree

12 files changed

+541
-0
lines changed
  • released/packages
    • coq-metacoq/coq-metacoq.1.3.4+8.20
    • coq-metacoq-common/coq-metacoq-common.1.3.4+8.20
    • coq-metacoq-erasure/coq-metacoq-erasure.1.3.4+8.20
    • coq-metacoq-erasure-plugin/coq-metacoq-erasure-plugin.1.3.4+8.20
    • coq-metacoq-pcuic/coq-metacoq-pcuic.1.3.4+8.20
    • coq-metacoq-quotation/coq-metacoq-quotation.1.3.4+8.20
    • coq-metacoq-safechecker/coq-metacoq-safechecker.1.3.4+8.20
    • coq-metacoq-safechecker-plugin/coq-metacoq-safechecker-plugin.1.3.4+8.20
    • coq-metacoq-template/coq-metacoq-template.1.3.4+8.20
    • coq-metacoq-template-pcuic/coq-metacoq-template-pcuic.1.3.4+8.20
    • coq-metacoq-translations/coq-metacoq-translations.1.3.4+8.20
    • coq-metacoq-utils/coq-metacoq-utils.1.3.4+8.20

12 files changed

+541
-0
lines changed
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,39 @@
1+
opam-version: "2.0"
2+
maintainer: "[email protected]"
3+
homepage: "https://metacoq.github.io/metacoq"
4+
dev-repo: "git+https://github.com/MetaCoq/metacoq.git#main"
5+
bug-reports: "https://github.com/MetaCoq/metacoq/issues"
6+
authors: ["Abhishek Anand <[email protected]>"
7+
"Danil Annenkov <[email protected]>"
8+
"Simon Boulier <[email protected]>"
9+
"Cyril Cohen <[email protected]>"
10+
"Yannick Forster <[email protected]>"
11+
"Jason Gross <[email protected]>"
12+
"Fabian Kunze <[email protected]>"
13+
"Meven Lennon-Bertrand <[email protected]>"
14+
"Kenji Maillard <[email protected]>"
15+
"Gregory Malecha <[email protected]>"
16+
"Jakob Botsch Nielsen <[email protected]>"
17+
"Matthieu Sozeau <[email protected]>"
18+
"Nicolas Tabareau <[email protected]>"
19+
"Théo Winterhalter <[email protected]>"
20+
]
21+
license: "MIT"
22+
build: [
23+
["bash" "./configure.sh"]
24+
[make "-j" "%{jobs}%" "-C" "common"]
25+
]
26+
install: [
27+
[make "-C" "common" "install"]
28+
]
29+
depends: [
30+
"coq-metacoq-utils" {= version}
31+
]
32+
synopsis: "The common library of Template Coq and PCUIC"
33+
description: """
34+
MetaCoq is a meta-programming framework for Coq.
35+
"""
36+
url {
37+
src: "https://github.com/MetaCoq/metacoq/archive/refs/tags/v1.3.4-8.20.tar.gz"
38+
checksum: "sha512=fb3997e2e07e9c33c293aabcc06b8e69785a9c2ebdcd4d48f77e1eb09698da6ed1770127022843f89322cf8f78289acd67c860e1a2d9186d5703191ccd088429"
39+
}
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,48 @@
1+
opam-version: "2.0"
2+
maintainer: "[email protected]"
3+
homepage: "https://metacoq.github.io/metacoq"
4+
dev-repo: "git+https://github.com/MetaCoq/metacoq.git#main"
5+
bug-reports: "https://github.com/MetaCoq/metacoq/issues"
6+
authors: ["Abhishek Anand <[email protected]>"
7+
"Danil Annenkov <[email protected]>"
8+
"Simon Boulier <[email protected]>"
9+
"Cyril Cohen <[email protected]>"
10+
"Yannick Forster <[email protected]>"
11+
"Jason Gross <[email protected]>"
12+
"Fabian Kunze <[email protected]>"
13+
"Meven Lennon-Bertrand <[email protected]>"
14+
"Kenji Maillard <[email protected]>"
15+
"Gregory Malecha <[email protected]>"
16+
"Jakob Botsch Nielsen <[email protected]>"
17+
"Matthieu Sozeau <[email protected]>"
18+
"Nicolas Tabareau <[email protected]>"
19+
"Théo Winterhalter <[email protected]>"
20+
]
21+
license: "MIT"
22+
build: [
23+
["bash" "./configure.sh"]
24+
[make "-j" "%{jobs}%" "-C" "erasure-plugin"]
25+
]
26+
install: [
27+
[make "-C" "erasure-plugin" "install"]
28+
]
29+
depends: [
30+
"coq-metacoq-template-pcuic" {= version}
31+
"coq-metacoq-erasure" {= version}
32+
]
33+
synopsis: "Implementation and verification of an erasure procedure for Coq"
34+
description: """
35+
MetaCoq is a meta-programming framework for Coq.
36+
37+
The Erasure module provides a complete specification of Coq's so-called
38+
\"extraction\" procedure, starting from the PCUIC calculus and targeting
39+
untyped call-by-value lambda-calculus.
40+
41+
The `erasure` function translates types and proofs in well-typed terms
42+
into a dummy `tBox` constructor, following closely P. Letouzey's PhD
43+
thesis.
44+
"""
45+
url {
46+
src: "https://github.com/MetaCoq/metacoq/archive/refs/tags/v1.3.4-8.20.tar.gz"
47+
checksum: "sha512=fb3997e2e07e9c33c293aabcc06b8e69785a9c2ebdcd4d48f77e1eb09698da6ed1770127022843f89322cf8f78289acd67c860e1a2d9186d5703191ccd088429"
48+
}
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,48 @@
1+
opam-version: "2.0"
2+
maintainer: "[email protected]"
3+
homepage: "https://metacoq.github.io/metacoq"
4+
dev-repo: "git+https://github.com/MetaCoq/metacoq.git#main"
5+
bug-reports: "https://github.com/MetaCoq/metacoq/issues"
6+
authors: ["Abhishek Anand <[email protected]>"
7+
"Danil Annenkov <[email protected]>"
8+
"Simon Boulier <[email protected]>"
9+
"Cyril Cohen <[email protected]>"
10+
"Yannick Forster <[email protected]>"
11+
"Jason Gross <[email protected]>"
12+
"Fabian Kunze <[email protected]>"
13+
"Meven Lennon-Bertrand <[email protected]>"
14+
"Kenji Maillard <[email protected]>"
15+
"Gregory Malecha <[email protected]>"
16+
"Jakob Botsch Nielsen <[email protected]>"
17+
"Matthieu Sozeau <[email protected]>"
18+
"Nicolas Tabareau <[email protected]>"
19+
"Théo Winterhalter <[email protected]>"
20+
]
21+
license: "MIT"
22+
build: [
23+
["bash" "./configure.sh"]
24+
[make "-j" "%{jobs}%" "-C" "erasure"]
25+
]
26+
install: [
27+
[make "-C" "erasure" "install"]
28+
]
29+
depends: [
30+
"coq-metacoq-safechecker" {= version}
31+
"coq-metacoq-template-pcuic" {= version}
32+
]
33+
synopsis: "Implementation and verification of an erasure procedure for Coq"
34+
description: """
35+
MetaCoq is a meta-programming framework for Coq.
36+
37+
The Erasure module provides a complete specification of Coq's so-called
38+
\"extraction\" procedure, starting from the PCUIC calculus and targeting
39+
untyped call-by-value lambda-calculus.
40+
41+
The `erasure` function translates types and proofs in well-typed terms
42+
into a dummy `tBox` constructor, following closely P. Letouzey's PhD
43+
thesis.
44+
"""
45+
url {
46+
src: "https://github.com/MetaCoq/metacoq/archive/refs/tags/v1.3.4-8.20.tar.gz"
47+
checksum: "sha512=fb3997e2e07e9c33c293aabcc06b8e69785a9c2ebdcd4d48f77e1eb09698da6ed1770127022843f89322cf8f78289acd67c860e1a2d9186d5703191ccd088429"
48+
}
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,43 @@
1+
opam-version: "2.0"
2+
maintainer: "[email protected]"
3+
homepage: "https://metacoq.github.io/metacoq"
4+
dev-repo: "git+https://github.com/MetaCoq/metacoq.git#main"
5+
bug-reports: "https://github.com/MetaCoq/metacoq/issues"
6+
authors: ["Abhishek Anand <[email protected]>"
7+
"Danil Annenkov <[email protected]>"
8+
"Simon Boulier <[email protected]>"
9+
"Cyril Cohen <[email protected]>"
10+
"Yannick Forster <[email protected]>"
11+
"Jason Gross <[email protected]>"
12+
"Fabian Kunze <[email protected]>"
13+
"Meven Lennon-Bertrand <[email protected]>"
14+
"Kenji Maillard <[email protected]>"
15+
"Gregory Malecha <[email protected]>"
16+
"Jakob Botsch Nielsen <[email protected]>"
17+
"Matthieu Sozeau <[email protected]>"
18+
"Nicolas Tabareau <[email protected]>"
19+
"Théo Winterhalter <[email protected]>"
20+
]
21+
license: "MIT"
22+
build: [
23+
["bash" "./configure.sh"]
24+
[make "-j" "%{jobs}%" "-C" "pcuic"]
25+
]
26+
install: [
27+
[make "-C" "pcuic" "install"]
28+
]
29+
depends: [
30+
"coq-metacoq-common" {= version}
31+
]
32+
synopsis: "A type system equivalent to Coq's and its metatheory"
33+
description: """
34+
MetaCoq is a meta-programming framework for Coq.
35+
36+
The PCUIC module provides a cleaned-up specification of Coq's typing algorithm along
37+
with a certified typechecker for it. This module includes the standard metatheory of
38+
PCUIC: Weakening, Substitution, Confluence and Subject Reduction are proven here.
39+
"""
40+
url {
41+
src: "https://github.com/MetaCoq/metacoq/archive/refs/tags/v1.3.4-8.20.tar.gz"
42+
checksum: "sha512=fb3997e2e07e9c33c293aabcc06b8e69785a9c2ebdcd4d48f77e1eb09698da6ed1770127022843f89322cf8f78289acd67c860e1a2d9186d5703191ccd088429"
43+
}
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,53 @@
1+
opam-version: "2.0"
2+
maintainer: "[email protected]"
3+
homepage: "https://metacoq.github.io/metacoq"
4+
dev-repo: "git+https://github.com/MetaCoq/metacoq.git#main"
5+
bug-reports: "https://github.com/MetaCoq/metacoq/issues"
6+
authors: ["Abhishek Anand <[email protected]>"
7+
"Danil Annenkov <[email protected]>"
8+
"Simon Boulier <[email protected]>"
9+
"Cyril Cohen <[email protected]>"
10+
"Yannick Forster <[email protected]>"
11+
"Jason Gross <[email protected]>"
12+
"Fabian Kunze <[email protected]>"
13+
"Meven Lennon-Bertrand <[email protected]>"
14+
"Kenji Maillard <[email protected]>"
15+
"Gregory Malecha <[email protected]>"
16+
"Jakob Botsch Nielsen <[email protected]>"
17+
"Matthieu Sozeau <[email protected]>"
18+
"Nicolas Tabareau <[email protected]>"
19+
"Théo Winterhalter <[email protected]>"
20+
]
21+
license: "MIT"
22+
build: [
23+
["bash" "./configure.sh"]
24+
[make "-j" "%{jobs}%" "-C" "quotation"]
25+
]
26+
install: [
27+
[make "-C" "quotation" "install"]
28+
]
29+
depends: [
30+
"coq-metacoq-template" {= version}
31+
"coq-metacoq-pcuic" {= version}
32+
"coq-metacoq-template-pcuic" {= version}
33+
]
34+
synopsis: "Gallina quotation functions for Template Coq"
35+
description: """
36+
MetaCoq is a meta-programming framework for Coq.
37+
38+
The Quotation module is geared at providing functions `□T → □□T` for
39+
`□T := Ast.term` (currently implemented) and for `□T := { t : Ast.term
40+
& Σ ;;; [] |- t : T }` (still in the works). Currently `Ast.term →
41+
Ast.term` and `(Σ ;;; [] |- t : T) → Ast.term` functions are provided
42+
for Template and PCUIC terms, in `MetaCoq.Quotation.ToTemplate.All`
43+
and `MetaCoq.Quotation.ToPCUIC.All`. Proving well-typedness is still
44+
a work in progress.
45+
46+
Ultimately the goal of this development is to prove that `□` is a lax monoidal
47+
semicomonad (a functor with `cojoin : □T → □□T` that codistributes over `unit`
48+
and `×`), which is sufficient for proving Löb's theorem.
49+
"""
50+
url {
51+
src: "https://github.com/MetaCoq/metacoq/archive/refs/tags/v1.3.4-8.20.tar.gz"
52+
checksum: "sha512=fb3997e2e07e9c33c293aabcc06b8e69785a9c2ebdcd4d48f77e1eb09698da6ed1770127022843f89322cf8f78289acd67c860e1a2d9186d5703191ccd088429"
53+
}
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,48 @@
1+
opam-version: "2.0"
2+
maintainer: "[email protected]"
3+
homepage: "https://metacoq.github.io/metacoq"
4+
dev-repo: "git+https://github.com/MetaCoq/metacoq.git#main"
5+
bug-reports: "https://github.com/MetaCoq/metacoq/issues"
6+
authors: ["Abhishek Anand <[email protected]>"
7+
"Danil Annenkov <[email protected]>"
8+
"Simon Boulier <[email protected]>"
9+
"Cyril Cohen <[email protected]>"
10+
"Yannick Forster <[email protected]>"
11+
"Jason Gross <[email protected]>"
12+
"Fabian Kunze <[email protected]>"
13+
"Meven Lennon-Bertrand <[email protected]>"
14+
"Kenji Maillard <[email protected]>"
15+
"Gregory Malecha <[email protected]>"
16+
"Jakob Botsch Nielsen <[email protected]>"
17+
"Matthieu Sozeau <[email protected]>"
18+
"Nicolas Tabareau <[email protected]>"
19+
"Théo Winterhalter <[email protected]>"
20+
]
21+
license: "MIT"
22+
build: [
23+
["bash" "./configure.sh"]
24+
[make "-j" "%{jobs}%" "-C" "safechecker-plugin"]
25+
]
26+
install: [
27+
[make "-C" "safechecker-plugin" "install"]
28+
]
29+
depends: [
30+
"coq-metacoq-template-pcuic" {= version}
31+
"coq-metacoq-safechecker" {= version}
32+
]
33+
synopsis: "Implementation and verification of an erasure procedure for Coq"
34+
description: """
35+
MetaCoq is a meta-programming framework for Coq.
36+
37+
The Erasure module provides a complete specification of Coq's so-called
38+
\"extraction\" procedure, starting from the PCUIC calculus and targeting
39+
untyped call-by-value lambda-calculus.
40+
41+
The `erasure` function translates types and proofs in well-typed terms
42+
into a dummy `tBox` constructor, following closely P. Letouzey's PhD
43+
thesis.
44+
"""
45+
url {
46+
src: "https://github.com/MetaCoq/metacoq/archive/refs/tags/v1.3.4-8.20.tar.gz"
47+
checksum: "sha512=fb3997e2e07e9c33c293aabcc06b8e69785a9c2ebdcd4d48f77e1eb09698da6ed1770127022843f89322cf8f78289acd67c860e1a2d9186d5703191ccd088429"
48+
}
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,42 @@
1+
opam-version: "2.0"
2+
maintainer: "[email protected]"
3+
homepage: "https://metacoq.github.io/metacoq"
4+
dev-repo: "git+https://github.com/MetaCoq/metacoq.git#main"
5+
bug-reports: "https://github.com/MetaCoq/metacoq/issues"
6+
authors: ["Abhishek Anand <[email protected]>"
7+
"Danil Annenkov <[email protected]>"
8+
"Simon Boulier <[email protected]>"
9+
"Cyril Cohen <[email protected]>"
10+
"Yannick Forster <[email protected]>"
11+
"Jason Gross <[email protected]>"
12+
"Fabian Kunze <[email protected]>"
13+
"Meven Lennon-Bertrand <[email protected]>"
14+
"Kenji Maillard <[email protected]>"
15+
"Gregory Malecha <[email protected]>"
16+
"Jakob Botsch Nielsen <[email protected]>"
17+
"Matthieu Sozeau <[email protected]>"
18+
"Nicolas Tabareau <[email protected]>"
19+
"Théo Winterhalter <[email protected]>"
20+
]
21+
license: "MIT"
22+
build: [
23+
["bash" "./configure.sh"]
24+
[make "-j" "%{jobs}%" "-C" "safechecker"]
25+
]
26+
install: [
27+
[make "-C" "safechecker" "install"]
28+
]
29+
depends: [
30+
"coq-metacoq-pcuic" {= version}
31+
]
32+
synopsis: "Implementation and verification of safe conversion and typechecking algorithms for Coq"
33+
description: """
34+
MetaCoq is a meta-programming framework for Coq.
35+
36+
The SafeChecker modules provides a correct implementation of
37+
weak-head reduction, conversion and typechecking of Coq definitions and global environments.
38+
"""
39+
url {
40+
src: "https://github.com/MetaCoq/metacoq/archive/refs/tags/v1.3.4-8.20.tar.gz"
41+
checksum: "sha512=fb3997e2e07e9c33c293aabcc06b8e69785a9c2ebdcd4d48f77e1eb09698da6ed1770127022843f89322cf8f78289acd67c860e1a2d9186d5703191ccd088429"
42+
}
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,39 @@
1+
opam-version: "2.0"
2+
maintainer: "[email protected]"
3+
homepage: "https://metacoq.github.io/metacoq"
4+
dev-repo: "git+https://github.com/MetaCoq/metacoq.git#main"
5+
bug-reports: "https://github.com/MetaCoq/metacoq/issues"
6+
authors: ["Abhishek Anand <[email protected]>"
7+
"Danil Annenkov <[email protected]>"
8+
"Simon Boulier <[email protected]>"
9+
"Cyril Cohen <[email protected]>"
10+
"Yannick Forster <[email protected]>"
11+
"Jason Gross <[email protected]>"
12+
"Fabian Kunze <[email protected]>"
13+
"Meven Lennon-Bertrand <[email protected]>"
14+
"Kenji Maillard <[email protected]>"
15+
"Gregory Malecha <[email protected]>"
16+
"Jakob Botsch Nielsen <[email protected]>"
17+
"Matthieu Sozeau <[email protected]>"
18+
"Nicolas Tabareau <[email protected]>"
19+
"Théo Winterhalter <[email protected]>"
20+
]
21+
license: "MIT"
22+
build: [
23+
["bash" "./configure.sh"]
24+
[make "-j" "%{jobs}%" "-C" "template-pcuic"]
25+
]
26+
install: [
27+
[make "-C" "template-pcuic" "install"]
28+
]
29+
depends: [
30+
"coq-metacoq-template" {= version}
31+
"coq-metacoq-pcuic" {= version}
32+
]
33+
synopsis: "Translations between Template Coq and PCUIC and proofs of correctness"
34+
description: """
35+
"""
36+
url {
37+
src: "https://github.com/MetaCoq/metacoq/archive/refs/tags/v1.3.4-8.20.tar.gz"
38+
checksum: "sha512=fb3997e2e07e9c33c293aabcc06b8e69785a9c2ebdcd4d48f77e1eb09698da6ed1770127022843f89322cf8f78289acd67c860e1a2d9186d5703191ccd088429"
39+
}

0 commit comments

Comments
 (0)