aboutsummaryrefslogtreecommitdiffhomepage
path: root/dev/ci
Commit message (Collapse)AuthorAge
* fix iris-lambda-rust CIGravatar Ralf Jung2018-04-18
|
* Merge PR #7242: Update the CI branch for Equations.Gravatar Gaëtan Gilbert2018-04-17
|\
| * Update the CI branch for Equations.Gravatar Théo Zimmermann2018-04-13
| |
* | Overlay for econstr in Evd.Gravatar Gaëtan Gilbert2018-04-13
|/
* Merge PR #6454: [econstr] Flag to make `to_constr` fail if its output ↵Gravatar Pierre-Marie Pédrot2018-04-13
|\ | | | | | | contains evars
* \ Merge PR #6809: Improve shell scriptsGravatar Michael Soegtrop2018-04-08
|\ \
| * | Improve shell scriptsGravatar zapashcanon2018-04-05
| | |
* | | [api] Move some types to their proper module.Gravatar Emilio Jesus Gallego Arias2018-04-02
|/ / | | | | | | | | | | | | | | | | | | | | | | We solve some modularity and type duplication problems by moving types to a better place. In particular: - We move tactics types from `Misctypes` to `Tactics` as this is their proper module an single user [with LTAC]. - We deprecate aliases in `Tacexpr` to such tactic types. cc: #6512
| * [econstr] Forbid calling `to_constr` in open terms.Gravatar Emilio Jesus Gallego Arias2018-03-31
|/ | | | | | | | | | | | | | | | | | | | | | | | We forbid calling `EConstr.to_constr` on terms that are not evar-free, as to progress towards enforcing the invariant that `Constr.t` is evar-free. [c.f. #6308] Due to compatibility constraints we provide an optional parameter to `to_constr`, `abort` which can be used to overcome this restriction until we fix all parts of the code. Now, grepping for `~abort:false` should return the questionable parts of the system. Not a lot of places had to be fixed, some comments: - problems with the interface due to `Evd/Constr` [`Evd.define` being the prime example] do seem real! - inductives also look bad with regards to `Constr/EConstr`. - code in plugins needs work. A notable user of this "feature" is `Obligations/Program` that seem to like to generate kernel-level entries with free evars, then to scan them and workaround this problem by generating constants.
* Remove outdated patch from ci-sfGravatar Jasper Hugunin2018-03-29
|
* [ssreflect] Fix module scoping problems due to packing and mli files.Gravatar Emilio Jesus Gallego Arias2018-03-10
| | | | | | | | | | | | | | | | | | | | Unfortunately, mli-only files cannot be included in packs, so we have the weird situation that the scope for `Tacexpr` is wrong. So we cannot address the module as `Ltac_plugin.Tacexpr` but it lives in the global namespace instead. This creates problem when using other modular build/packing strategies [such as #6857] This could be indeed considered a bug in the OCaml compiler. In order to remedy this situation we face two choices: - leave the module out of the pack (!) - create an implementation for the module I chose the second solution as it seems to me like the most sensible choice. cc: #6512.
* [located] Push inner locations in `reference` to a CAst.t node.Gravatar Emilio Jesus Gallego Arias2018-03-09
| | | | | | | | | | | | | | The `reference` type contains some ad-hoc locations in its constructors, but there is no reason not to handle them with the standard attribute container provided by `CAst.t`. An orthogonal topic to this commit is whether the `reference` type should contain a location or not at all. It seems that many places would become a bit clearer by splitting `reference` into non-located `reference` and `lreference`, however some other places become messier so we maintain the current status-quo for now.
* [located] More work towards using CAst.tGravatar Emilio Jesus Gallego Arias2018-03-09
| | | | | | | | | | | We continue with the work of #402 and #6745 and update most of the remaining parts of the AST: - module declarations - intro patterns - top-level sentences Now, parsed documents should be full annotated by `CAst` nodes.
* Merge PR #6775: Allow using cumulativity without forcing strict constraints.Gravatar Maxime Dénès2018-03-09
|\
| * Overlay for Elpi.Gravatar Gaëtan Gilbert2018-03-09
| |
* | Add an overlay for Equations and Ltac2.Gravatar Pierre-Marie Pédrot2018-03-09
|/
* Merge PR #6881: [windows] support -addon in build scriptGravatar Maxime Dénès2018-03-08
|\
| * build: win: turn off build/installation of gnu MakeGravatar Enrico Tassi2018-03-06
| |
* | Merge PR #6511: [econstr] Continue consolidation of EConstr API under `interp`.Gravatar Maxime Dénès2018-03-04
|\ \
* \ \ Merge PR #6676: [proofview] goals come with a stateGravatar Maxime Dénès2018-03-04
|\ \ \
| | | * build: win: addon bignumsGravatar Enrico Tassi2018-03-02
| |_|/ |/| |
| | * [econstr] Continue consolidation of EConstr API under `interp`.Gravatar Emilio Jesus Gallego Arias2018-02-28
| |/ |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This commit was motivated by true spurious conversions arising in my `to_constr` debug branch. The changes here need careful review as the tradeoffs are subtle and still a lot of clean up remains to be done in `vernac/*`. We have opted for penalize [minimally] the few users coming from true `Constr`-land, but I am sure we can tweak code in a much better way. In particular, it is not clear if internalization should take an `evar_map` even in the cases where it is not triggered, see the changes under `plugins` for a good example. Also, the new return type of `Pretyping.understand` should undergo careful review. We don't touch `Impargs` as it is not clear how to proceed, however, the current type of `compute_implicits_gen` looks very suspicious as it is called often with free evars. Some TODOs are: - impargs was calling whd_all, the Econstr equivalent can be either + Reductionops.whd_all [which does refolding and no sharing] + Reductionops.clos_whd_flags with all as a flag.
* | [ast] Improve precision of Ast location recognition in serialization.Gravatar Emilio Jesus Gallego Arias2018-02-22
| | | | | | | | | | | | | | | | | | We follow the suggestions in #402 and turn uses of `Loc.located` in `vernac` into `CAst.t`. The impact should be low as this change mostly affects top-level vernaculars. With this change, we are even closer to automatically map a text document to its AST in a programmatic way.
| * overlay for ltac2 and EquationsGravatar Enrico Tassi2018-02-20
| |
* | ci: add elpiGravatar Enrico Tassi2018-02-19
|/
* Merge PR #6706: ci-common: guess CI_BRANCH for local buildsGravatar Maxime Dénès2018-02-12
|\
* \ Merge PR #6610: Points to Flocq official repository.Gravatar Maxime Dénès2018-02-07
|\ \
* \ \ Merge PR #6686: Kernel/checker reduction cleanups around projection unfoldingGravatar Maxime Dénès2018-02-07
|\ \ \
| | | * ci-common: guess CI_BRANCH for local buildsGravatar Gaëtan Gilbert2018-02-07
| |_|/ |/| |
| | * Points to Flocq official repository.Gravatar Théo Zimmermann2018-02-05
| |/ |/| | | | | Following comment at https://github.com/coq/coq/pull/6596#issuecomment-358246528.
| * Add overlay for equations (nf_beta takes an env)Gravatar Gaëtan Gilbert2018-02-05
| |
* | Merge PR #6654: CI: Run coqchk on IrisGravatar Maxime Dénès2018-02-05
|\ \ | |/ |/|
| * CI: Run coqchk on IrisGravatar Ralf Jung2018-01-31
| |
* | Merge PR #6641: ci-compcert.sh: use default value for NJOBS when installing ↵Gravatar Maxime Dénès2018-01-31
|\ \ | | | | | | | | | menhir.
* \ \ Merge PR #6535: Cleanup name-binding structure for fresh evar name generation.Gravatar Maxime Dénès2018-01-31
|\ \ \ | |_|/ |/| |
| | * Put default value for NJOBS in ci-common.Gravatar Gaëtan Gilbert2018-01-30
| |/ |/|
| * Adding an overlay for Equations.Gravatar Pierre-Marie Pédrot2018-01-30
| |
* | Merge PR #6568: Cleanup scriptsGravatar Maxime Dénès2018-01-23
|\ \
| * | Source basic overlay before user overlays.Gravatar Gaëtan Gilbert2018-01-16
| | |
| * | Cleanup shell expansions and quoting.Gravatar Gaëtan Gilbert2018-01-16
| |/
* | Merge PR #6483: Strong invariants in polymorphic definitionsGravatar Maxime Dénès2018-01-12
|\ \
| * | Adding a custom Travis overlay for HoTT.Gravatar Pierre-Marie Pédrot2018-01-11
| | |
* | | Merge PR #6557: First stab at documenting the test suite.Gravatar Maxime Dénès2018-01-11
|\ \ \ | |/ / |/| |
| * | First stab at documenting the test suite.Gravatar Jasper Hugunin2018-01-06
| |/
* / Normalize Windows installer names.Gravatar Théo Zimmermann2018-01-04
|/
* Merge PR #6493: [API] remove large file containing duplicate interfacesGravatar Maxime Dénès2017-12-29
|\
* \ Merge PR #6405: Remove the local polymorphic flag hack.Gravatar Maxime Dénès2017-12-29
|\ \
| | * overlay for #6493Gravatar Enrico Tassi2017-12-27
| |/ |/|
* | Merge PR #6102: Fix #5998: AppVeyor package building is currently failingGravatar Maxime Dénès2017-12-27
|\ \
| | * Add equations overlay.Gravatar Maxime Dénès2017-12-27
| |/ |/|