aboutsummaryrefslogtreecommitdiffhomepage
path: root/dev
Commit message (Collapse)AuthorAge
* Merge PR#622: Change the default flag value for Refine.refineGravatar Maxime Dénès2017-06-14
|\
* \ Merge PR#771: [travis overlay] Partially Revert 013c0232953f1f58Gravatar Maxime Dénès2017-06-14
|\ \
* | | Temporary overlays because fewer plugins are loaded at startup.Gravatar Maxime Dénès2017-06-14
| | |
* | | [travis] overlay for fiat-crypto (a Require Import FunInd)Gravatar Pierre Letouzey2017-06-14
| | |
* | | [travis] overlays for CompCert and VST (an extra Require Export FunInd)Gravatar Pierre Letouzey2017-06-14
| | |
* | | [travis] fix Software Foundation (one added Require Extraction)Gravatar Pierre Letouzey2017-06-14
| | |
* | | [travis] fix CoLoR by inserting some Require Import FunIndGravatar Pierre Letouzey2017-06-14
| | |
* | | Temporary overlays for bignums.Gravatar Maxime Dénès2017-06-14
| | |
* | | Merge PR#498: Bignums as a separate opam packageGravatar Maxime Dénès2017-06-14
|\ \ \
* \ \ \ Merge PR#766: Fix ocamldebug for the APIGravatar Maxime Dénès2017-06-13
|\ \ \ \
* \ \ \ \ Merge PR#714: Print feature Proof-of-Concept (episode 2)Gravatar Maxime Dénès2017-06-13
|\ \ \ \ \
| | | | | * Dualize the unsafe flag of refine into typecheck and make it mandatory.Gravatar Pierre-Marie Pédrot2017-06-13
| | | | | |
| | | * | | [travis] overlay for cornGravatar Pierre Letouzey2017-06-13
| | | | | |
| | | * | | [travis] extra test ci-bignums (+factorize other scripts)Gravatar Pierre Letouzey2017-06-13
| | | | | |
| | | * | | [travis] overlay + extra deps for math-classes (and formal-topology)Gravatar Pierre Letouzey2017-06-13
| | | | | |
| | | | | * Documenting the change of default flag value of Refine.refine.Gravatar Pierre-Marie Pédrot2017-06-13
| | | | | |
| | | * | | [travis] adapt CoLoR compilation to depend on the bignum packageGravatar Pierre Letouzey2017-06-13
| |_|/ / / |/| | | |
* | | | | Merge PR#764: Point ci-hott at a newer version of HoTTGravatar Maxime Dénès2017-06-13
|\ \ \ \ \ | |_|_|_|/ |/| | | |
* | | | | Merge PR#715: Add coq-dpdgraph ciGravatar Maxime Dénès2017-06-12
|\ \ \ \ \
| | | | | * [travis overlay] Partially Revert 013c0232953f1f58Gravatar Jason Gross2017-06-12
| |_|_|_|/ |/| | | | | | | | | I've pushed commits which add `-bypass-API` to bedrock in the proper way, so these overlays are no longer needed
* | | | | Merge PR#718: API cleanup: aliasesGravatar Maxime Dénès2017-06-12
|\ \ \ \ \
* | | | | | Temporary overlay, waiting for upstream PR merges.Gravatar Maxime Dénès2017-06-12
| | | | | |
* | | | | | add overlaysGravatar Matej Košík2017-06-12
| | | | | |
| | | | | * Fix ocamldebug for the APIGravatar Gaëtan Gilbert2017-06-12
| |_|_|_|/ |/| | | |
| | | * | Point ci-hott at a newer version of HoTTGravatar Jason Gross2017-06-11
| |_|/ / |/| | |
| * | | Remove (useless) aliases from the API.Gravatar Matej Košík2017-06-10
| | | |
| | * | Mirror dpdgraph's travis test more accuratelyGravatar Jason Gross2017-06-08
| | | |
| | * | Remove coq-dpdgraph overlayGravatar Jason Gross2017-06-08
| | | |
* | | | Merge branch 'v8.6'Gravatar Pierre-Marie Pédrot2017-06-08
|\ \ \ \ | |/ / / |/| | |
* | | | Remove overlay.Gravatar Maxime Dénès2017-06-08
| | | |
* | | | add overlaysGravatar Matej Košík2017-06-07
| | | |
* | | | Put all plugins behind an "API".Gravatar Matej Kosik2017-06-07
| | | |
* | | | Overlay.Gravatar Maxime Dénès2017-06-06
| | | |
* | | | Remove some overlays.Gravatar Maxime Dénès2017-06-06
| | | |
* | | | Overlays.Gravatar Maxime Dénès2017-06-06
| | | |
* | | | Merge PR#723: [travis] [fiat] Test also fiat-core.Gravatar Maxime Dénès2017-06-06
|\ \ \ \
* \ \ \ \ Merge PR#590: A more explicit algebraic type for evars of kind MatchingVar + ↵Gravatar Maxime Dénès2017-06-05
|\ \ \ \ \ | | | | | | | | | | | | | | | | | | a flag suspectingly renamed in a clearer way
| | | | | * Added support for a side effect on constants in reduction functions.Gravatar Thomas Sibut-Pinote2017-06-04
| |_|_|_|/ |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This exports two functions: - declare_reduction_effect: to declare a hook to be applied when some constant are visited during the execution of some reduction functions (primarily cbv, but also cbn, simpl, hnf, ...). - set_reduction_effect: to declare a constant on which a given effect hook should be called. Developed jointly by Thomas Sibut-Pinote and Hugo Herbelin. Added support for printing effect in functions of tacred.ml.
| | | | * Add an overlay for coq-dpdgraph for 8.7Gravatar Jason Gross2017-06-02
| | | | |
| | | | * Add coq-dpdgraph CIGravatar Jason Gross2017-06-02
| |_|_|/ |/| | |
| | * | [travis] [fiat] Test also fiat-core.Gravatar Emilio Jesus Gallego Arias2017-06-02
| |/ / |/| | | | | | | | I didn't rename the test file to `fiat` as IMHO it is not worth the noise.
* | | Merge PR#696: Trunk+cleanup constr of globalGravatar Maxime Dénès2017-06-01
|\ \ \
| | * | Adding overlay for math-comp.Gravatar Hugo Herbelin2017-05-31
| | | |
* | | | Creating a module Nameops.Name extending module Names.Name.Gravatar Hugo Herbelin2017-05-31
| |/ / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This module collects the functions of Nameops which are about Name.t and somehow standardize or improve their name, resulting in particular from discussions in working group. Note the use of a dedicated exception rather than a failwith for Nameops.Name.out. Drawback of the approach: one needs to open Nameops, or to use long prefix Nameops.Name.
* | | Merge PR#687: Gitlab CIGravatar Maxime Dénès2017-05-29
|\ \ \
| | * | Cleanup: removal of constr_of_global.Gravatar Matthieu Sozeau2017-05-29
| |/ / |/| | | | | | | | | | | | | | Constrintern.pf_global returns a global_reference, not a constr, adapt plugins accordingly, properly registering universes where necessary.
* | | Merge PR#512: [cleanup] Unify all calls to the error function.Gravatar Maxime Dénès2017-05-29
|\ \ \
| | * | Gitlab CIGravatar Gaëtan Gilbert2017-05-28
| | | |
| * | | [cleanup] Unify all calls to the error function.Gravatar Emilio Jesus Gallego Arias2017-05-27
| |/ / | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This is the continuation of #244, we now deprecate `CErrors.error`, the single entry point in Coq is `user_err`. The rationale is to allow for easier grepping, and to ease a future cleanup of error messages. In particular, we would like to systematically classify all error messages raised by Coq and be sure they are properly documented. We restore the two functions removed in #244 to improve compatibility, but mark them deprecated.
* / / [coqlib] Move `Coqlib` to `library/`.Gravatar Emilio Jesus Gallego Arias2017-05-27
|/ / | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | We move Coqlib to library in preparation for the late binding of Gallina-level references. Placing `Coqlib` in `library/` is convenient as some components such as pretyping need to depend on it. By moving we lose the ability to locate references by syntactic abbreviations, but IMHO it makes to require ML code to refer to a true constant instead of an abbreviation/notation. Unfortunately this change means that we break the `Coqlib` API (providing a compatibility function is not possible), however we do so for a good reason. The main changes are: - move `Coqlib` to `library/`. - remove reference -> term from `Coqlib`. In particular, clients will have different needs with regards to universes/evar_maps, so we force them to call the (not very safe) `Universes.constr_of_global` explicitly so the users are marked. - move late binding of impossible case from `Termops` to `pretying/Evarconv`. Remove hook. - `Coqlib.find_reference` doesn't support syntactic abbreviations anymore. - remove duplication of `Coqlib` code in `Program`. - remove duplication of `Coqlib` code in `Ltac.Rewrite`. - A special note about bug 5066 and commit 6e87877 . This case illustrates the danger of duplication in the code base; the solution chosen there was to transform the not-found anomaly into an error message, however the general policy was far from clear. The long term solution is indeed make `find_reference` emit `Not_found` and let the client handle the error maybe non-fatally. (so they can test for constants.