aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* [ci] Test coqchk on the CompCert target.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.
* \ \ 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
|\ \ \ \ \
| | | * | | 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.
| | | * Fix (partial) #4878: option to stop autodeclaring axiom as instance.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
|\ \ \ \ \ \ \ \ \ \ \ \ \ \ \ \
| | | | | | | | | | | | | | | | * A cosmetic standardization: adding a space in g_constr.ml4.Gravatar Hugo Herbelin2017-11-27
| | | | | | | | | | | | | | | | |
| | | | | | | | | | | | | | | | * Releasing level "11" of "pattern".Gravatar Hugo Herbelin2017-11-27
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Was introduced in 0917ce7c to fix #4272, but it seems that we can fix it by just merging levels 10 and 11. This prevents the worry of fixing the associativity of level 11 to left in 0917ce7c.
| | | | | | | | | | | | | | | | * Fixing associativity registered for level 10.Gravatar Hugo Herbelin2017-11-27
| |_|_|_|_|_|_|_|_|_|_|_|_|_|_|/ |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Apparently a long-standing bug, coupled with a pattern/constr associativity inconsistency introduced while fixing another pattern/constr level inconsistency (bug #4272, 0917ce7c).
| | | | | | | | | | | | | * | | [api] Remove aliases of `Evar.t`Gravatar Emilio Jesus Gallego Arias2017-11-26
| |_|_|_|_|_|_|_|_|_|_|_|/ / / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | There don't really bring anything, we also correct some minor nits with the printing function.
| | | | | | | | | | | | | | * Overlay for stronger restrict_universe_context.Gravatar Gaëtan Gilbert2017-11-25
| | | | | | | | | | | | | | |
| | | | | | | | | | | | | | * Restrict universe context when declaring constants in obligations.Gravatar Gaëtan Gilbert2017-11-25
| | | | | | | | | | | | | | |
| | | | | | | | | | | | * | | Updating the current official writing of OCaml, updating Camlp4->Camlp5.Gravatar Hugo Herbelin2017-11-25
| |_|_|_|_|_|_|_|_|_|_|/ / / |/| | | | | | | | | | | | |
| | | | | | | | | | | | | * Fix #5347: unify declaration of axioms with and without bound univs.Gravatar Gaëtan Gilbert2017-11-25
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Note that this makes the following syntax valid: Axiom foo@{i} bar : Type@{i}. (ie putting a universe declaration on the first axiom in the list, the declaration then holds for the whole list).
| | | | | | | | | | | | | * Fix interpretation of global universes in univdecl constraints.Gravatar Gaëtan Gilbert2017-11-25
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Also nicer error when the constraints are impossible.
| | | | | | | | | | | | | * Forbid repeated names in universe binders.Gravatar Gaëtan Gilbert2017-11-25
| | | | | | | | | | | | | |
| | | | | | | | | | | | | * Universe binders survive sections, modules and compilation.Gravatar Gaëtan Gilbert2017-11-25
| | | | | | | | | | | | | |
| | | | | | | | | | | | | * Allow local universe renaming in Print.Gravatar Gaëtan Gilbert2017-11-25
| | | | | | | | | | | | | |
| | | | | | | | | | | | | * Make restrict_universe_context stronger.Gravatar Gaëtan Gilbert2017-11-25
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This fixes BZ#5717. Also add a test and fix a changed test.
| | | | | | | | | | | | | * Fix obligations handling of universes anticipating stronger restrictGravatar Matthieu Sozeau2017-11-25
| | | | | | | | | | | | | |
| | | | | | * | | | | | | | [lib] Generalize Control.timeout type.Gravatar Emilio Jesus Gallego Arias2017-11-24
| |_|_|_|_|/ / / / / / / / |/| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | We also remove some internal implementation details from the mli file, there due historical reasons.
| | | | | | | | | * | | | Use Evarutil.has_undefined_evars for tactic has_evar.Gravatar Gaëtan Gilbert2017-11-24
| |_|_|_|_|_|_|_|/ / / / |/| | | | | | | | | | |
| | | | | | | | | | | * In close_proof only check univ decls with the restricted context.Gravatar Gaëtan Gilbert2017-11-24
| | | | | | | | | | | |
| | | | | | | | | | | * Use Entries.constant_universes_entry more.Gravatar Gaëtan Gilbert2017-11-24
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This reduces conversions between ContextSet/UContext and encodes whether we are polymorphic by which constructor we use rather than using some boolean.
| | | | | | | | | | | * When declaring constants/inductives use ContextSet if monomorphic.Gravatar Gaëtan Gilbert2017-11-24
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Also use constant_universes_entry instead of a bool flag to indicate polymorphism in ParameterEntry. There are a few places where we convert back to ContextSet because check_univ_decl returns a UContext, this could be improved.
| | | | | | | | | | | * restrict_universe_context: do not prune named universes.Gravatar Gaëtan Gilbert2017-11-24
| | | | | | | | | | | |
| | | | | | | | | | | * Fix defining non primitive projections with abstracted universes.Gravatar Gaëtan Gilbert2017-11-24
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | I think this only affects printing (in the new test you would get [Var (0)] when printing runwrap) but is still ugly.