aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* Declarative mode: remaining goals are "given up" when closing blocks.Gravatar Arnaud Spiwack2015-04-22
| | | Restores the intended behaviour from v8.3 and earlier.
* Fixing non exhaustive pattern-matching.Gravatar Hugo Herbelin2015-04-22
|
* Test for #4198 (appcontext in return clause of match).Gravatar Hugo Herbelin2015-04-22
|
* More precise numbers about Benjamin's fix for the VM.Gravatar Maxime Dénès2015-04-22
|
* Update CHANGESGravatar Matthieu Sozeau2015-04-22
|
* Do not use list concatenation when gluing streams together, just mark them ↵Gravatar Guillaume Melquiond2015-04-22
| | | | | | | | | | | | as glued. Possible improvement: rotate using the left children in the glue function, so that the iter function becomes mostly tail-recursive. Drawback: two allocations per glue instead of a single one. This commit makes the following command go from 7.9s to 3.0s: coqtop <<< "Require Import BigZ ZBinary Reals OrdersEx. Time SearchPattern _." | tail -n 1
* Remove some spurious spaces in generated Makefiles.Gravatar Guillaume Melquiond2015-04-22
|
* STM: print trace on "anomaly, no safe id attached"Gravatar Enrico Tassi2015-04-21
|
* Fixing #4198 (looking for subterms also in the return clause of match).Gravatar Hugo Herbelin2015-04-21
| | | | | This is actually not so perfect because of the lambdas in the return clause which we would not like to look in.
* Fixing #3383 (a "return" clause without an "in" clause is not enoughGravatar Hugo Herbelin2015-04-21
| | | | for being able to interpret a "match" as a constr pattern).
* Fixing #3376 and #4191 (wrong index of maximally-inserted implicit argumentGravatar Hugo Herbelin2015-04-21
| | | | in the presence of let-ins).
* Some dead code.Gravatar Hugo Herbelin2015-04-21
|
* Remove spurious ".v" from warning message.Gravatar Guillaume Melquiond2015-04-20
|
* Change magic numbers.Gravatar Matthieu Sozeau2015-04-20
|
* Inlining "fun" and "forall" tokens in parser, so that alternative notations forGravatar Hugo Herbelin2015-04-20
| | | | them (e.g. "fun ... ⇒ ...") factor well (see #2268).
* Slightly more efficient implementation of the logic monad.Gravatar Pierre-Marie Pédrot2015-04-19
| | | | We just inline the state in the iolist: less closures makes the GC happier.
* 8.5beta2 release.Gravatar Matthieu Sozeau2015-04-17
|
* Extra fix to 934761875 and f4ee7ee31e4 on optimizing Import of severalGravatar Hugo Herbelin2015-04-17
| | | | libraries at once (see #4193).
* Fixing a few typos + some uniformization of writing in doc.Gravatar Hugo Herbelin2015-04-17
|
* No longer add dev/ to the LoadPath, only to the ML path.Gravatar Guillaume Melquiond2015-04-17
| | | | | | This patch should get rid of the following warning: Invalid character '-' in identifier "v8-syntax".
* Ensuring purity of datastructures in the API.Gravatar Pierre-Marie Pédrot2015-04-16
|
* Test for bug #4190.Gravatar Pierre-Marie Pédrot2015-04-16
|
* Fixing bug #4190.Gravatar Pierre-Marie Pédrot2015-04-16
| | | | | | | | | | The solution is a bit ugly. In order for two tactic notations identifiers not to be confused by the inclusion from two distinct modules, we embed the name of the source module in the identifiers. This may still fail if the same module is included twice with two distinct parameters, but this should not be possible thanks to the fact any definition in there will forbid the inclusion, for it would be repeated. People including twice the same empty module otherwise probably deserve whatever will arise from it.
* configure: fix paths on cygwinGravatar Enrico Tassi2015-04-16
| | | | | | | | | | | | | | | | | | | | | | Long story short: Filname.concat and other OCaml provided functions to be "cross platform" don't work for us for two reasons: 1. their behavior is fixed when one compiles ocaml, not when one runs it 2. the build system of Coq is unix only What is wrong with 1 is that if one compiles ocaml for windows without requiring cygwin.dll (a good thing, since you don't need to have cygwin to run ocaml) then the runtime always uses \ as dir_sep, no matter if you are running ocaml from a cygwin shell. If you use \ as a dir separaton in cygwin command lines, without going trough the cygpath "mangler", then things go wrong. The second point is that the makefiles we have need a unix like environment (e.g. we call sed). So you can't compile Coq without cygwin, unless you use a different build system, that is not what we support (1 build system is enough work already, IMO). To sum up: Running coq/ocaml requires no cygwin, comipling coq requires a unix like shell, hence paths shall be unix like in configure/build stuff.
* Remove dirty debug printing from funind.Gravatar Maxime Dénès2015-04-15
|
* Documenting the recommandation of toplevel-only commands.Gravatar Pierre-Marie Pédrot2015-04-15
|
* Function now supports puniveresGravatar jforest2015-04-14
|
* better debug in recdefGravatar jforest2015-04-14
|
* Cleaning up the implementation of search entries in Hints.Gravatar Pierre-Marie Pédrot2015-04-14
|
* Opaque implementation of auto tactics.Gravatar Pierre-Marie Pédrot2015-04-14
| | | | | | We provide an eliminator ensuring that the AST will be used to build a tactic, so that we can stuff arbitrary things inside. An escape function is also provided for backward compatibility.
* correction of a bug reported by Tristan CrolardGravatar jforest2015-04-13
|
* Program: Do not reduce obligation types preemptively, only atGravatar Matthieu Sozeau2015-04-13
| | | | definition time. The obligation tactic or user can still choose to do so.
* Remove declarations of matched variables in change as an extension ofGravatar Matthieu Sozeau2015-04-13
| | | | the context... overlooked by my last commit. Fixes relation-algebra.
* More documented representation of hint objects.Gravatar Pierre-Marie Pédrot2015-04-13
|
* Fixing bug #4186.Gravatar Pierre-Marie Pédrot2015-04-13
|
* Making the hint entry type opaque.Gravatar Pierre-Marie Pédrot2015-04-12
|
* Fix compilation broken by Matthieu's last commit.Gravatar Pierre Letouzey2015-04-10
| | | | | | | | Btw, also unset the READABLE_ML4 option, which probably caused this issue. No, we normally do *not* want to see the internals of .ml generated out of a .ml4 (except during some specific debug sessions). It is *so* easy otherwise to edit the wrong .ml by mistake and forget to edit the original .ml4.
* Fix #3590 for good this time, by changing the API, change's argument nowGravatar Matthieu Sozeau2015-04-10
| | | | | | takes a variable substitution for matched variables in the (lhs) pattern, and uses the existing ist structure to pretype the rhs correcly, without having to deal with the volatile evars.
* Test for bug #3199.Gravatar Pierre-Marie Pédrot2015-04-10
|
* Eauto hints respect their priority. Fixes bug #3199.Gravatar Pierre-Marie Pédrot2015-04-10
| | | | | | | | This patch changes the semantics of eauto w.r.t. to extern hints, so it may break some code out there. There is no compatibility flag because this is a real bug, and we do not really want the users to depend on this. Moreover, there are still some fishy parts in the current implementation that should be rewritten for the next release.
* Making the hints for the auto tactics private.Gravatar Pierre-Marie Pédrot2015-04-10
| | | | | | They are all generated by the Hints module, and making them purely opaque is not worthwhile because we project them a lot. This ensures that they all get generated following a uniform process.
* Better test-suite files, removing reliance on admit.Gravatar Matthieu Sozeau2015-04-09
|
* Fix declarations of instances to perform restriction of universeGravatar Matthieu Sozeau2015-04-09
| | | | instances as definitions and lemmas do (fixes bug# 4121).
* Add test-suite file for bug #4120.Gravatar Matthieu Sozeau2015-04-09
|
* Really fix constr_of_pattern and bugs #3590 and #4120 byGravatar Matthieu Sozeau2015-04-09
| | | | | removing all evars appearing in the constr (or their types, recursively) from the evar_map.
* Strengthen minimization: it shouldn't set a universe u to a max if itGravatar Matthieu Sozeau2015-04-09
| | | | has a strict upper bound.
* Remove evars in the type of _unnammed_ metas in pattern_of_constr (fixes ↵Gravatar Matthieu Sozeau2015-04-09
| | | | QuicksortComplexity).
* Prove [map_ext] using [map_ext_in].Gravatar Nickolai Zeldovich2015-04-09
| | | | Since [map_ext_in] is more general, no need to have the same proof twice.
* Add a [map_ext_in] lemma to List.v.Gravatar Nickolai Zeldovich2015-04-09
| | | | | | Slightly broader version of the existing [map_ext]: two [map] expressions are equal if their respective functions agree on all arguments that are in the list being mapped.
* JSON extraction: make explicit each group of mutually-recursive fixpointsGravatar Nickolai Zeldovich2015-04-09
|