aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
* More sharing in Logic, together with some code cleaning.Gravatar Pierre-Marie Pédrot2014-02-21
* Optimization in kernel/vars.ml: directly allocate a fixed-size block in theGravatar Pierre-Marie Pédrot2014-02-20
* CoqIDE: when coqtop misbehaves kill it properly (no zombie)Gravatar Enrico Tassi2014-02-17
* [nanoPG]: emacs like copy/pasteGravatar Enrico Tassi2014-02-17
* Removing non-marshallable data from the Agram constructor. Instead ofGravatar Pierre-Marie Pédrot2014-02-16
* fast correction of bug #3234Gravatar Julien Forest2014-02-14
* TC: honor the use_typeclasses flag in pretypingGravatar Enrico Tassi2014-02-12
* Made Pre_env.lazy_val opaque.Gravatar Pierre-Marie Pédrot2014-02-11
* Timeout and Set Default Timeout fixed (closes: #3229)Gravatar Enrico Tassi2014-02-10
* STM: fix valid_id coming from Qed errorsGravatar Enrico Tassi2014-02-10
* STM: when a worker is canceled mark the proof as brokenGravatar Enrico Tassi2014-02-10
* STM: be conservative w.r.t. proofs containing global side effectsGravatar Enrico Tassi2014-02-10
* fake_ide: ported to spawnGravatar Enrico Tassi2014-02-10
* Tentative fixup for the previous commit. It seems I have broken somethingGravatar Pierre-Marie Pédrot2014-02-10
* Small optimizations in Closure:Gravatar Pierre-Marie Pédrot2014-02-09
* Less dependencies in Omega.Gravatar Pierre-Marie Pédrot2014-02-08
* FinFun.v: results about injective/surjective/bijective fonctions over finite ...Gravatar Pierre Letouzey2014-02-07
* Tactic extensions do not need to be classified by the STM, asGravatar Pierre-Marie Pédrot2014-02-05
* The constructor tactic now returns several successes.Gravatar Pierre-Marie Pédrot2014-02-04
* Tracking memory misallocation by trying to improve sharing.Gravatar Pierre-Marie Pédrot2014-02-03
* Allocation-friendly mapping functions in Nametab.Gravatar Pierre-Marie Pédrot2014-02-03
* Allocation friendly map-handling functions in Dag.Gravatar Pierre-Marie Pédrot2014-02-03
* Fixing backtrace reporting.Gravatar Pierre-Marie Pédrot2014-02-02
* Fixing bug #3226.Gravatar Pierre-Marie Pédrot2014-02-02
* Removing the [Require "file"] syntax.Gravatar Pierre-Marie Pédrot2014-02-02
* In Ltac's exact tactic: avoid checking the type of the term twice.Gravatar Arnaud Spiwack2014-01-31
* Typos in comment.Gravatar Arnaud Spiwack2014-01-31
* Coqmktop without Sys.command, changes in ./configure -*byteflags optionsGravatar Pierre Letouzey2014-01-30
* Relaunch all Unix.waitpid when they ended with EINTRGravatar Pierre Letouzey2014-01-30
* CUnix: enriched (get_extension, sys_command, waitpid_non_intr) + cleanedGravatar Pierre Letouzey2014-01-30
* Mltop: explicitly qualify calls to CUnixGravatar Pierre Letouzey2014-01-30
* CString: avoid redefining is_subGravatar Pierre Letouzey2014-01-30
* Remove useless Xml_utilsGravatar Pierre Letouzey2014-01-30
* Get rid of two utility files, obsolete now that configure is a .mlGravatar Pierre Letouzey2014-01-30
* clib.mllib: remove duplicated Flags entryGravatar Pierre Letouzey2014-01-30
* G_xml: remove some duplication in error fonctionsGravatar Pierre Letouzey2014-01-30
* G_xml: protect against some possible Not_foundGravatar Pierre Letouzey2014-01-30
* Load implemented in CoqIDE/STM (closes: #3223)Gravatar Enrico Tassi2014-01-30
* STM + CoqIDE: stop_worker message and UIGravatar Enrico Tassi2014-01-30
* Work around for bug in threads + blocking io streamlinedGravatar Enrico Tassi2014-01-30
* STM: worker sends back to master the last valid stateGravatar Enrico Tassi2014-01-30
* STM: tell the user if the master is recomputing states validated by workersGravatar Enrico Tassi2014-01-30
* Fixing backtrace handling here and there.Gravatar Pierre-Marie Pédrot2014-01-30
* Using Map.smartmap whenever deemed useful.Gravatar Pierre-Marie Pédrot2014-01-29
* Adding a smartmap[i] operator to maps.Gravatar Pierre-Marie Pédrot2014-01-29
* Fixing dependent inversion. Some exceptions were not caught by the tacticGravatar Pierre-Marie Pédrot2014-01-28
* Abstracting away coercion indexes in Classops.Gravatar Pierre-Marie Pédrot2014-01-27
* Coercions: avoid imperative data structureGravatar Enrico Tassi2014-01-26
* -schedule-vi-checking ported to spawnGravatar Enrico Tassi2014-01-26
* CoqIDE: command line for extra coqtop "flags"Gravatar Enrico Tassi2014-01-26