Skip to content

Commit

Permalink
Test CI
Browse files Browse the repository at this point in the history
  • Loading branch information
proux01 committed Jul 21, 2024
1 parent 0d87ad7 commit 1123afc
Show file tree
Hide file tree
Showing 9 changed files with 4,283 additions and 0 deletions.
3,649 changes: 3,649 additions & 0 deletions .github/workflows/nix-action-coq-master.yml

Large diffs are not rendered by default.

223 changes: 223 additions & 0 deletions .nix/config.nix
Original file line number Diff line number Diff line change
@@ -0,0 +1,223 @@
with builtins; with (import <nixpkgs> {}).lib;
{
## DO NOT CHANGE THIS
format = "1.0.0";
## unless you made an automated or manual update
## to another supported format.

## The attribute to build from the local sources,
## either using nixpkgs data or the overlays located in `.nix/coq-overlays`
## Will determine the default main-job of the bundles defined below
attribute = "stdlib";

## If you want to select a different attribute (to build from the local sources as well)
## when calling `nix-shell` and `nix-build` without the `--argstr job` argument
# shell-attribute = "{{nix_name}}";

## Maybe the shortname of the library is different from
## the name of the nixpkgs attribute, if so, set it here:
# pname = "{{shortname}}";

## Lists the dependencies, phrased in terms of nix attributes.
## No need to list Coq, it is already included.
## These dependencies will systematically be added to the currently
## known dependencies, if any more than Coq.
## /!\ Remove this field as soon as the package is available on nixpkgs.
## /!\ Manual overlays in `.nix/coq-overlays` should be preferred then.
# buildInputs = [ ];

## Indicate the relative location of your _CoqProject
## If not specified, it defaults to "_CoqProject"
coqproject = "theories/_CoqProject";

## Cachix caches to use in CI
## Below we list some standard ones
cachix.coq = {};
cachix.math-comp = {};
# cachix.coq-community = {};

## If you have write access to one of these caches you can
## provide the auth token or signing key through a secret
## variable on GitHub. Then, you should give the variable
## name here. For instance, coq-community projects can use
## the following line instead of the one above:
cachix.coq-community.authToken = "CACHIX_AUTH_TOKEN";

## Or if you have a signing key for a given Cachix cache:
# cachix.my-cache.signingKey = "CACHIX_SIGNING_KEY"

## Note that here, CACHIX_AUTH_TOKEN and CACHIX_SIGNING_KEY
## are the names of secret variables. They are set in
## GitHub's web interface.

## select an entry to build in the following `bundles` set
## defaults to "default"
default-bundle = "coq-master";

## write one `bundles.name` attribute set per
## alternative configuration
## When generating GitHub Action CI, one workflow file
## will be created per bundle
bundles = let
## In some cases, light overrides are not available/enough
## in which case you can use either
# coqPackages.<coq-pkg>.overrideAttrs = o: <overrides>;
## or a "long" overlay to put in `.nix/coq-overlays
## you may use `nix-shell --run fetchOverlay <coq-pkg>`
## to automatically retrieve the one from nixpkgs
## if it exists and is correctly named/located

## You can override Coq and other coqPackages
## through the following attribute
## If <ocaml-pkg> does not support light overrides,
## you may use `overrideAttrs` or long overlays
## located in `.nix/ocaml-overlays`
## (there is no automation for this one)
# ocamlPackages.<ocaml-pkg>.override.version = "x.xx";

## You can also override packages from the nixpkgs toplevel
# <nix-pkg>.override.overrideAttrs = o: <overrides>;
## Or put an overlay in `.nix/overlays`

## you may mark a package as a main CI job (one to take deps and
## rev deps from) as follows
# coqPackages.<main-pkg>.main-job = true;
## by default the current package and its shell attributes are main jobs

## you may mark a package as a CI job as follows
# coqPackages.<another-pkg>.job = "test";
## It can then built through
## nix-build --argstr bundle "default" --arg job "test";
## in the absence of such a directive, the job "another-pkg" will
## is still available, but will be automatically included in the CI
## via the command genNixActions only if it is a dependency or a
## reverse dependency of a job flagged as "main-job" (see above).

## Run on push on following branches (default [ "master" ])
# push-branches = [ "master" "branch2" ];

master = [
"stdlib"
"mathcomp"
"fourcolor"
"odd-order"
"mathcomp-zify"
"mathcomp-finmap"
"mathcomp-bigenough"
"mathcomp-analysis"
# TODO unimath
# TODO unicoq
# "math-classes" -> overlay
# "corn" -> overlay
"stdpp"
"iris"
# "autosubst" -> overlay
# TODO tests from iris/examples
# TODO hott
# "coqhammer" -> overlay
# "flocq" -> overlay
# TODO coq-performance-tests
# TODO coq-tools
"coquelicot"
"compcert"
"vst"
# TODO cross-crypto
# TODO rewriter
# TODO fiat_parsers
# TODO fiat_crypto_legacy
# TODO fiat_crypto
# TODO rupicola
# TODO bedrock2
# TODO coqutil
# TODO kami
# TODO riscv_coq
# TODO color
"bignums"
"coqprime"
# TODO bbv
# TODO coinduction
# "coq-elpi" -> overlay
"hierarchy-builder"
# TODO engine bench
# TODO fcsl_pcm
# "coq-ext-lib" -> overlay
"simple-io"
"QuickChick"
# TODO reduction_effects
# TODO menhirlib
# TODO neural_net_interp
# "aac-tactics" -> overlay
"paco"
# TODO itree
# TODO itree_io
"ceres"
"parsec"
# TODO json
# TODO async_test
# TODO http
"paramcoq"
# "relation-algebra" -> overlay
"StructTact"
"InfSeqExt"
"Cheerios"
"Verdi"
# TODO verdi-raft
# TODO stdlib2
# TODO argosy
# TODO atbr
# TODO perennial
# TODO sf
# TODO Coqtail
"deriving"
# TODO vscoq (is vscoq-language-server enough?)
"category-theory"
"itauto"
"mathcomp-word"
# TODO jasmin
# TODO coq-lean-importer
# TODO smtcoq_trakt
# TODO stalmarck
# TODO tactician
# TODO ltac2_compiler
# TODO waterproof
# TODO autosubst OCaml
];
coq-master = [
"dpdgraph"
"smtcoq"
"trakt"
];
main = [
"coq-lsp"
# "equations" -> overlay
"metacoq"
"serapi"
];
common-bundles = listToAttrs (forEach master (p:
{ name = p; value.override.version = "master"; }))
// listToAttrs (forEach coq-master (p:
{ name = p; value.override.version = "coq-master"; }))
// listToAttrs (forEach main (p:
{ name = p; value.override.version = "main"; }))
// {
coq-elpi.override.version = "proux01:split_stdlib";
mathcomp.override.version = "proux01:split_stdlib";
# tlc.override.version = "master-for-coq-ci"; -> overlay
tlc.override.version = "proux01:split_stdlib";
flocq.override.version = "split_stdlib";
coq-ext-lib.override.version = "split_stdlib";
aac-tactics.override.version = "split_stdlib";
coqhammer.override.version = "proux01:split_stdlib";
math-classes.override.version = "split_stdlib";
corn.override.version = "split_stdlib";
equations.override.version = "proux01:split_stdlib";
autosubst.override.version = "split_stdlib";
relation-algebra.override.version = "proux01:split_stdlib";
};
in {
"coq-master".coqPackages = common-bundles // {
coq.override.version = "proux01:split_stdlib";
};
"coq-master".ocamlPackages = { elpi.override.version = "1.19.2"; };
};
}
1 change: 1 addition & 0 deletions .nix/coq-nix-toolbox.nix
Original file line number Diff line number Diff line change
@@ -0,0 +1 @@
"3170ff10f08b5767b9763c05e71d7481b5fdcc30"
Loading

0 comments on commit 1123afc

Please sign in to comment.