aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* [configure] fix detection of `md5sum`Gravatar Vincent Laporte2017-12-04
|
* Merge PR #736: [ci] Test coqchk on the CompCert target.Gravatar Maxime Dénès2017-12-01
|\
* \ Merge PR #6256: CI: better ocaml warning checksGravatar Maxime Dénès2017-12-01
|\ \
* \ \ Merge PR #6276: Coqchk accepts filenamesGravatar Maxime Dénès2017-12-01
|\ \ \
* \ \ \ Merge PR #6233: [proof] [api] Rename proof types in preparation for ↵Gravatar Maxime Dénès2017-12-01
|\ \ \ \ | | | | | | | | | | | | | | | functionalization.
* \ \ \ \ Merge PR #1049: Remove obsolete localityGravatar Maxime Dénès2017-11-30
|\ \ \ \ \
* \ \ \ \ \ Merge PR #6244: [lib] [api] Introduce record for `object_prefix`Gravatar Maxime Dénès2017-11-30
|\ \ \ \ \ \
| | | | | | * [ci] Test coqchk on the CompCert target.Gravatar Théo Zimmermann2017-11-30
| | | | | | |
* | | | | | | Merge PR #6274: Attempt to fix inversion disregarding singleton types (fixes ↵Gravatar Maxime Dénès2017-11-30
|\ \ \ \ \ \ \ | |_|_|_|_|_|/ |/| | | | | | | | | | | | | #3125)
* | | | | | | Merge PR #6269: [ci] [vst] Shorten compilation time to avoid Travis timeouts.Gravatar Maxime Dénès2017-11-30
|\ \ \ \ \ \ \
* \ \ \ \ \ \ \ Merge PR #6193: Fix (partial) #4878: option to stop autodeclaring axiom as ↵Gravatar Maxime Dénès2017-11-30
|\ \ \ \ \ \ \ \ | | | | | | | | | | | | | | | | | | | | | | | | | | | instance.
| | | | | * | | | Remove "obsolete_locality" and fix STM vernac classification.Gravatar Maxime Dénès2017-11-29
| |_|_|_|/ / / / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | We remove deprecated syntax "Coercion Local" and such, and seize the opportunity to refactor some code around vernac_expr. We also do a small fix on the STM classification, which didn't know about Let Fixpoint and Let CoFixpoint. This is a preliminary step for the work on attributes.
| | | | * | | | [lib] [api] Introduce record for `object_prefix`Gravatar Emilio Jesus Gallego Arias2017-11-29
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This is a minor cleanup adding a record in a try to structure the state living in `Lib`.
| | | | | * | | [proof] [api] Rename proof types in preparation for functionalization.Gravatar Emilio Jesus Gallego Arias2017-11-29
| |_|_|_|/ / / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | In particular `Proof_global.t` will become a first class object for the upper parts of the system in a next commit.
* | | | | | | Merge PR #6271: Add PR backport script.Gravatar Maxime Dénès2017-11-29
|\ \ \ \ \ \ \
* \ \ \ \ \ \ \ Merge PR #6253: Fixing inconsistent associativity of level 10 in the table ↵Gravatar Maxime Dénès2017-11-29
|\ \ \ \ \ \ \ \ | | | | | | | | | | | | | | | | | | | | | | | | | | | of levels
* \ \ \ \ \ \ \ \ Merge PR #6199: [vernac] Uniformize type of vernac interpretation.Gravatar Maxime Dénès2017-11-29
|\ \ \ \ \ \ \ \ \
| | | | | | | | * | coq_makefile: pass filenames to coqchkGravatar Ralf Jung2017-11-29
| | | | | | | | | |
| | | | | | | | * | Documenting the possibility to pass filenames to coqchk.Gravatar Pierre-Marie Pédrot2017-11-29
| | | | | | | | | |
| | | | | | | | * | Allow to pass physical files to coqchk.Gravatar Pierre-Marie Pédrot2017-11-29
| | | | | | | | | |
| | | | | | * | | | In injection/inversion, consider all template-polymorphic types as injectable.Gravatar Hugo Herbelin2017-11-28
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | In particular singleton inductive types are considered injectable, even in the absence of the option "Set Keep Proof Equalities". This fixes #3125 (and #4560, #6273).
| | | | | | * | | | Adding a variant get_truncation_family_of of get_sort_family_of.Gravatar Hugo Herbelin2017-11-28
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This function returns InProp or InSet for inductive types only when the inductive type has been explicitly truncated to Prop or (impredicative) Set. For instance, singleton inductive types and small (predicative) inductive types are not truncated and hence in Type.
| | | | | | * | | | Moving non-recursive function sort_family_of out of the retype block of ↵Gravatar Hugo Herbelin2017-11-28
| | | | | | |/ / / | | | | | | | | | | | | | | | | | | | | | | | | | | | recursive functions.
| | | | | | | * / Adding an interface file for checker/check.ml.Gravatar Pierre-Marie Pédrot2017-11-28
| |_|_|_|_|_|/ / |/| | | | | | |
| | | * | | | | Add PR backport script.Gravatar Théo Zimmermann2017-11-28
| |_|/ / / / / |/| | | | | |
| | | | * | | [ci] [vst] Shorten compilation time to avoid Travis timeouts.Gravatar Emilio Jesus Gallego Arias2017-11-28
| |_|_|/ / / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | We remove the progs target [examples] to save time, we still build the full library thou. I guess we can't do better for now unless we get some Travis subscription.
| | | | | * CI: use -byte-only in [warnings] jobs.Gravatar Gaëtan Gilbert2017-11-28
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This avoids mixing native and byte compilation as the debug printers are always byte compiled and the tools have no .byte rule, only the OCAMLBEST rule.
| | | | | * Fix native compute for byte compiled Coq.Gravatar Gaëtan Gilbert2017-11-28
| | | | | |
| | | * | | Fix (partial) #4878: option to stop autodeclaring axiom as instance.Gravatar Gaëtan Gilbert2017-11-28
| |_|/ / / |/| | | |
| | | | * Travis: do not build stdlib in [warnings] jobs.Gravatar Gaëtan Gilbert2017-11-28
| |_|_|/ |/| | |
* | | | Merge PR #6259: Add PR merge script.Gravatar Maxime Dénès2017-11-28
|\ \ \ \
| * | | | Add PR merge script.Gravatar Maxime Dénès2017-11-28
| | | | |
* | | | | Merge PR #1033: Universe binder improvementsGravatar Maxime Dénès2017-11-28
|\ \ \ \ \
* \ \ \ \ \ Merge PR #6235: Fixing failing mkdir in test-suite for coq-makefile.Gravatar Maxime Dénès2017-11-28
|\ \ \ \ \ \
* \ \ \ \ \ \ Merge PR #6248: [api] Remove aliases of `Evar.t`Gravatar Maxime Dénès2017-11-28
|\ \ \ \ \ \ \
* \ \ \ \ \ \ \ Merge PR #6246: Ref. Man.: Updating the current official writing of OCaml; ↵Gravatar Maxime Dénès2017-11-28
|\ \ \ \ \ \ \ \ | |_|_|_|_|_|_|/ |/| | | | | | | | | | | | | | | updating Camlp4->Camlp5.
| | | | | | * | [vernac] Adjust `interp` to pass polymorphic in the attributes.Gravatar Emilio Jesus Gallego Arias2017-11-27
| | | | | | | |
| | | | | | * | [vernac] Add polymorphic to the type of vernac interpration options.Gravatar Emilio Jesus Gallego Arias2017-11-27
| | | | | | | |
| | | | | | * | [vernac] Start to uniformize type of vernac interpretation.Gravatar Emilio Jesus Gallego Arias2017-11-27
| |_|_|_|_|/ / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | In particular, we put all the context in the atts structure, and generalize the type of the parameters of a vernac. I hope this helps people working on "attributes", my motivation is indeed having a more robust interpretation.
* | | | | | | Merge PR #6237: coq_makefile tests: build in easily removed temporary ↵Gravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ | |_|_|_|_|/ / |/| | | | | | | | | | | | | subdirectory.
* | | | | | | Merge PR #6242: Use Evarutil.has_undefined_evars for tactic has_evar.Gravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \
* \ \ \ \ \ \ \ Merge PR #6236: Fix coq-makefile ocamldoc call when configured with -annotate.Gravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ Merge PR #6207: [stm] Allow delayed constant in interactive mode.Gravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ \ Merge PR #6238: Fix deprecated syntax warning from vernacextend.mlp.Gravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ \ \ Merge PR #6241: [lib] Generalize Control.timeout type.Gravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ \ \ \ Merge PR #6228: Make byte on gitlab.Gravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ \ \ \ \ Merge PR #6226: Enhance votourGravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ \ \ \ \ \ Merge PR #6149: Update TimeFileMaker.py to correctly sort timing diffsGravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ \ \ \ \ \ \ Merge PR #6041: Protecting the printing of filenames with spaceGravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ \ \ \ \ \ \ \ Merge PR #6227: Linter: do not lint untracked files.Gravatar Maxime Dénès2017-11-27
|\ \ \ \ \ \ \ \ \ \ \ \ \ \ \ \