aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
...
* | | | | | | | | | | | | | | | | | 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)
| | | | | | | | * | | | | | | | | | | Add merlin in the dependencies of nix-shell only.Gravatar Théo Zimmermann2017-11-30
| |_|_|_|_|_|_|/ / / / / / / / / / / |/| | | | | | | | | | | | | | | | |
* | | | | | | | | | | | | | | | | | 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.
| | | | | | | | | | | | | | * | | | | Fix usage comment.Gravatar Théo Zimmermann2017-11-29
| | | | | | | | | | | | | | | | | | |
| | | | | | | | | | | | | | * | | | | This script apparently uses bash-specific features.Gravatar Théo Zimmermann2017-11-29
| | | | | | | | | | | | | | | | | | |
| | | | | | | | | | | | | | * | | | | Fix PR merge script.Gravatar Théo Zimmermann2017-11-29
| |_|_|_|_|_|_|_|_|_|_|_|_|/ / / / / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Was still relying on the existence of user-configured /pr/.
| | | | * | | | | | | | | | | | | | [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`.
| | | | | | | | | | | * | | | | | Forbid implicitly relative names in the checker.Gravatar Pierre-Marie Pédrot2017-11-29
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Before this patch, passing a mere identifier (without dots) to the checker would make it consider it as implicitly referring to a relative name. For instance, if passed "foo", it would have looked for "Bar.foo.vo" and "Qux.foo.vo" if those files were in the loadpath. This was quite ad-hoc. We remove this "feature" and require the user to always give either a filename or a fully qualified logical name.
| | | | | | | | | | | * | | | | | Mark the -I option in coqchk as deprecated and merge it with -Q.Gravatar Pierre-Marie Pédrot2017-11-29
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | It is not doing the same thing as coqtop, and the corresponding coqtop semantics is irrelevant in the checker as the latter does not rely on ML code.
| | | | | | | | | | | * | | | | | Add a -Q option to coqchck.Gravatar Pierre-Marie Pédrot2017-11-29
| | | | | | | |_|_|_|/ / / / / / | | | | | | |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | It has exactly the same effect as -R, because there is no such thing as implicit relativization for object files in coqchk, contrarily to what Require does in coqtop.
| | | | | * / | | | | | | | | | [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).
| | | | | | | | | | | * | | | | | | use \ocaml macro in new textGravatar Paul Steckler2017-11-28
| | | | | | | | | | | | | | | | | |
| | | | | | * | | | | | | | | | | | 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
| |_|_|_|_|_|/ / / / / / / / / / |/| | | | | | | | | | | | | | |
| | | | | | | | * | | | | | | | more complete not-fully-applied error messages, #6145Gravatar Paul Steckler2017-11-28
| | | | | | | | | | | | | | | |
| | | * | | | | | | | | | | | | Add PR backport script.Gravatar Théo Zimmermann2017-11-28
| |_|/ / / / / / / / / / / / / |/| | | | | | | | | | | | | |
| | | | | | | | | | | | | | * [toplevel] Properly redirect stdout on `Redirect` vernac.Gravatar Emilio Jesus Gallego Arias2017-11-28
| |_|_|_|_|_|_|_|_|_|_|_|_|/ |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Fixes #6130, it was a silly omission from a previous output refactoring. We redirect all channels as this was the implied semantics of the old command.
| | | | * | | | | | | | | | [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.
| | | | | | | | * | | | | Use safe demarshalling in the checker.Gravatar Pierre-Marie Pédrot2017-11-28
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Instead of relying on the OCaml demarshaller, which is not resilient against ill-formed data, we reuse the safe demarshaller from votour. This ensures that garbage files do not trigger memory violations.
| | | | | | | | * | | | | Use large arrays in the checker demarshaller.Gravatar Pierre-Marie Pédrot2017-11-28
| |_|_|_|_|_|_|/ / / / / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This allows to work around the size limitation of vanilla OCaml arrays on 32-bit platforms, which is rather easy to hit.
| | | | | * | | | | | | 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
| |_|_|/ / / / / / / |/| | | | | | | | |
| | | | | | | | * | Add alienclean target to remove compilation products with no source.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.
| | | | | | | | | * | | | allow :: and , as infix opsGravatar Paul Steckler2017-11-27
| | | | | | | | | | | | |
| | | | | | * | | | | | | [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.
| | | | | | | | | | * | Selecting which notation to print based on current stack of scope.Gravatar Hugo Herbelin2017-11-27
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | See discussion on coq-club starting on 23 August 2016. An open question: what priority to give to "abbreviations"?
| | | | | | | | | | * | Pre-isolating a notation test to avoid interferences.Gravatar Hugo Herbelin2017-11-27
| |_|_|_|_|_|_|_|_|/ / |/| | | | | | | | | |
| | | | | | | | | | * Adding overlay for ltac2.Gravatar Hugo Herbelin2017-11-27
| | | | | | | | | | |