aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* Qed: feedback when type checking is doneGravatar Enrico Tassi2013-12-24
| | | | | | To make this possible the state id has to reach the kernel. Hence definition_entry has an extra field, and many files had to be fixed.
* CoqIDE: new feedback "incomplete" to signal partial QedGravatar Enrico Tassi2013-12-24
|
* Future: optional greedy chainingGravatar Enrico Tassi2013-12-24
| | | | | | If a Future.computation is already a value v or an exception and is chained in a greedy way with a function f, then f v is executed immediately (or the exception is raised).
* cleanup warningGravatar Enrico Tassi2013-12-24
|
* Simplifying the use of hypinfos in Rewrite.Gravatar Pierre-Marie Pédrot2013-12-24
|
* Rewrite.ml: removing direction flag from hypinfo.Gravatar Pierre-Marie Pédrot2013-12-23
|
* Do not pass unification flags around in Rewrite.Gravatar Pierre-Marie Pédrot2013-12-22
|
* Slight code cleaning ensuring more static invariants in Rewrite.Gravatar Pierre-Marie Pédrot2013-12-22
|
* Adding -bt to coqc.Gravatar Pierre-Marie Pédrot2013-12-22
|
* Adding a finer-grained -bt flag to coqtop only triggering backtraces.Gravatar Pierre-Marie Pédrot2013-12-22
|
* Notation variables are now taken into account as possible ltac bound variablesGravatar Pierre-Marie Pédrot2013-12-22
| | | | when internalizing a term.
* Notations now accept the $(...)$ tactic-in-term syntax. They are resolved atGravatar Pierre-Marie Pédrot2013-12-22
| | | | internalization time.
* Notations can now accept dummy arguments. If ever a bound variable is notGravatar Pierre-Marie Pédrot2013-12-22
| | | | | | used, they are automatically flagged as only parsing. CAVEAT: unused arguments are not typechecked, because they are dropped before the interpretation phase.
* Test case for the buggy commutative cut subterm rule.Gravatar Maxime Dénès2013-12-21
|
* configure.ml: our configure script is now written in ML :-)Gravatar Pierre Letouzey2013-12-20
| | | | | | | | | | | | | | | | | | configure is now just a minimal wrapper around the new configure.ml. This configure.ml is runned with the same ocaml used during compilation, and starts with a #load "unix.cma". For now, this new configure script is meant to be 99% compatible with the old one. Known incompatibilities : the --foo option format (with two --) isn't supported anymore, use -foo options instead. Let me know if you encounter any other changes. Internals: - We use our own "run" command (based on Unix.create_process) to avoid relying on some specific shell (/bin/sh or cmd.exe). - We should have far less issues with filename quoting under windows since we almost never rely on (cygwin) shell anymore. This remains to be fully tested, though. - dev/ocamldebug-coq is slightly different now, to ease its generation
* Makefile.build: avoid a -ppGravatar Pierre Letouzey2013-12-20
|
* coqc: execvp is now available even on win32Gravatar Pierre Letouzey2013-12-20
|
* coqmktop without Unix (simpler all_subdirs)Gravatar Pierre Letouzey2013-12-20
|
* Remove unused Makefile lines about .elc compilationGravatar Pierre Letouzey2013-12-20
|
* Warning removalGravatar Pierre Boutillier2013-12-20
|
* List: Bug 3039 weaker requirement for fold symmetricGravatar Pierre Boutillier2013-12-20
|
* Coqdep always uses / as dir_sepGravatar Pierre Boutillier2013-12-20
|
* micromega: removal of spurious Export; addition of Lia.v encapsulating lia ↵Gravatar Frédéric Besson2013-12-20
| | | | and nia.
* Removing the useless pattern ident genarg.Gravatar Pierre-Marie Pédrot2013-12-19
|
* Using interp_genarg in tactic notations where possible, instead of an ad-hocGravatar Pierre-Marie Pédrot2013-12-19
| | | | interpreter.
* test-suite/output/Notations : evar number changeGravatar Pierre Boutillier2013-12-19
|
* Bad use of Obj.magic in interpretation of TacAlias arguments.Gravatar Pierre Boutillier2013-12-19
| | | | | | It triggered nonsensical behaviour of list-using tactic notation. Hopefully or not, nobody uses such notations out of the test-suite...
* Printing function for Stdargs in debuggerGravatar Pierre Boutillier2013-12-19
|
* Missing Fail in r16792Gravatar Pierre Boutillier2013-12-19
|
* test guard condition against feature incompatible with prop-extGravatar Bruno Barras2013-12-17
|
* Fix make install after 3e972b3ff8e532be233f70567c87512324c99b4eGravatar Pierre Boutillier2013-12-17
| | | | | Attempt to adapt .el files too. doc/refman/RefMan-uti.tex has still to be fixed.
* Merge branch 'trunk' of github.com:coq/coq into trunkGravatar Matthieu Sozeau2013-12-17
|\
* | Tentative fix of the guardedness checker by Christine and me. All stdlib and ↵Gravatar Matthieu Sozeau2013-12-17
| | | | | | | | test-suite pass.
| * Removing the need of evarmaps in constr internalization.Gravatar Pierre-Marie Pédrot2013-12-17
|/ | | | | | Actually, this was wrong, as evars should not appear until interpretation. Evarmaps were only passed around uselessly, and often fed with dummy or irrelevant values.
* Get rid of messages "emitting ..." when compiling .v filesGravatar Pierre Letouzey2013-12-16
| | | | | If these messages are still relevent to somebody, feel free to restore them in -debug or any non-default mode of your choice.
* A few fixes to the build system (mostly for ocamlbuild)Gravatar Pierre Letouzey2013-12-16
| | | | | | | | | | | | | | * vars.mli was mentionning Term instead of Constr, leading to a dep cycle * Having a file named toplevel/toplevel.ml isn't a good idea when we also have a toplevel/toplevel.mllib that ought to produce a toplevel.cma. We rename toplevel.ml into Coqloop.ml * Extra cleanup of toplevel.mllib : - Ppextra isn't anywhere around (?!) - Ppvernac was mentionned twice, and rather belongs to printing.mllib anyway - Vernacexpr is a .mli and shouldn't appear in an .mllib * During the link, printing.cma now comes after parsing.cma (Ppvernac uses Egramml) * A few extra -threads in ocamlbuild files (btw, it's a bit sad to need -thread for coqchk).
* Added test-suite for bug #2990.Gravatar Pierre-Marie Pédrot2013-12-16
|
* Dedicated inductive for return values of rewrite strategies.Gravatar Pierre-Marie Pédrot2013-12-16
|
* Do not overallocate closures' named environments in infos. Modifying the accessGravatar Pierre-Marie Pédrot2013-12-15
| | | | function is sufficient to skip the undefined variables.
* Do not compile coqide with -threadGravatar Pierre Boutillier2013-12-12
| | | | Coqide compiled with -thread seems to hang for ever at startup under MacOS
* Patch for supporting [From Xxx Require Yyy Zzz.]Gravatar Gregory Malecha2013-12-12
| | | | | | | | | | | | When using libraries I find it convenient (and future proof) to use fully qualified paths in many places. It would be nice to have a convenient short-hand for this so that you can: From Xxx Require Yyy Zzz. instead of having to type: Require Xxx.Yyy Xxx.Zzz. Signed-off-by: Pierre Boutillier <pierre.boutillier@ens-lyon.org>
* Better unification for [projT1] and [proj1_sig].Gravatar Jason Gross2013-12-12
| | | | | | | This way, [fun A (P : A -> Prop) (X : sigT P) => proj1_sig X] unifies with [fun A (P : A -> Prop) (X : sigT P) => projT1 X]. This closes Bug 3043.
* Generalize eq_proofs_unicityGravatar Jason Gross2013-12-12
| | | | | | | | | | | | | | | The generalizded version is eq_proofs_unicity_one_var. We preserve backwards compatibility, unless someone used nu_left_inv (which was defined as a Remark(!), but whose type depended on a number of Lets.) We could keep going in defining one variable variants, but I was lazy. I'm also not sure if we should be breaking backward compatiblity to generalize these theorems, if we should make separate files for the pointed versions, or if we should just have duplicate theorems in each file. (I'm also not sure if I should call it _one_var or _pointed or something else.) This closes Bug 3019.
* Documenting the tactic-in-term construction.Gravatar Pierre-Marie Pédrot2013-12-11
|
* Fix CoqIDE compilation under standard version of lablgtk2Gravatar Enrico Tassi2013-12-11
| | | | We use the win32 specific function only if WIN32 is defined
* Fixing backtrace registering of various tactic-related try-with blocks.Gravatar Pierre-Marie Pédrot2013-12-11
|
* Fix CoqIDE on windowsGravatar Enrico Tassi2013-12-10
|
* Renaming elisp files to avoid conflict with pg in distribs.Gravatar Pierre Courtieu2013-12-10
|
* Fix printing of Ltac's backtrace.Gravatar Arnaud Spiwack2013-12-09
| | | I used an exception wrapper to report Tactic failures. It had the consequence of making process_vernac_interp_error to look for the backtrace at the wrong place.
* Stylistic change.Gravatar Arnaud Spiwack2013-12-09
| | | I doubt [catching_error] is performance critical in any way. But it looked silly to allocate a block to [(inner_trace,e)] when [e] was known in advance (and was already named [e]).