aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel
Commit message (Expand)AuthorAge
* Updated all headers for 8.3 and trunkGravatar herbelin2010-07-24
* fixed (serious) bug #2353: non-recursive parameters of nested inductive types...Gravatar barras2010-07-16
* removed a potentially dangerous try ... with _ -> ...Gravatar barras2010-07-16
* Mod_typing: fix the content of the typ_expr_alg fieldGravatar letouzey2010-07-07
* Names: remove obsolete mod_self_idGravatar letouzey2010-06-23
* New script dev/tools/change-header to automatically update Coq files headers.Gravatar herbelin2010-06-22
* Added printing of recursive notations in cases pattern (supported by wish 2248).Gravatar herbelin2010-06-14
* Fixing spelling: pr_coma -> pr_commaGravatar herbelin2010-06-12
* "Improved" the form of the inferred type of "match" byGravatar herbelin2010-06-03
* fixed guard check with commutative cutsGravatar barras2010-05-20
* Mrec was not substituted correctlyGravatar barras2010-05-20
* Discontinue support for ocaml 3.09.*Gravatar letouzey2010-05-19
* Some ocamldoc comments + Fixing name of .coqrc.version file in refmanGravatar pboutill2010-05-18
* Applicative commutative cuts in Fixpoint guard conditionGravatar pboutill2010-05-18
* Removed $Id$ introduced inadvertently in r13005 (no more $Id$ since r12972)Gravatar herbelin2010-05-09
* Added a few informations about file lineages (for the most part in kernel)Gravatar herbelin2010-05-09
* "make source-doc" builds documentation of mli in html and pdf atGravatar pboutill2010-04-29
* After the approval of Bruno, here the patch for the checker.Gravatar soubiran2010-04-29
* Various minor improvements of comments in mli for ocamldocGravatar letouzey2010-04-29
* fixed bug #2224 (Error message in positivity check fixed)Gravatar vsiles2010-04-29
* Remove the svn-specific $Id$ annotationsGravatar letouzey2010-04-29
* Move from ocamlweb to ocamdoc to generate mli documentationGravatar pboutill2010-04-29
* Here comes the commit, announced long ago, of the new tactic engine.Gravatar aspiwack2010-04-22
* Fixed bug #2999 (destruct was not refreshing universes of what it generalized *)Gravatar herbelin2010-04-20
* In function "substitution_prefixed_by" the prefix test on module path Gravatar soubiran2010-04-19
* cf. 12945Gravatar soubiran2010-04-16
* Names.mli: double declaration of mind_modpathGravatar letouzey2010-04-16
* fixed confusion between number of cstr arguments and number of pattern variab...Gravatar barras2010-03-12
* introduced lazy computation of size info in the guard conditionGravatar barras2010-03-11
* Added a lazy evaluation of the composition of module substitutions. It improv...Gravatar soubiran2010-02-04
* fix commit 12706 + comments.Gravatar soubiran2010-02-03
* Small fix on module inclusion.Gravatar soubiran2010-02-02
* Various bug fix on recent features of the module system:Gravatar soubiran2010-01-19
* Variant !F M for functor application that does not honor the Inline declarationsGravatar letouzey2010-01-17
* Include can accept both Module and Module TypeGravatar letouzey2010-01-07
* Patch on subtyping check of opaque constants.Gravatar soubiran2010-01-06
* The following script was rasing an errorGravatar soubiran2010-01-04
* Fixing bug #2156 (non positive occurrence error message displayed "Rel"'s).Gravatar herbelin2009-12-30
* revert on commit r12553Gravatar barras2009-12-07
* declaremods.ml <--- code factoringGravatar soubiran2009-12-03
* two improvements of the guard condition:Gravatar barras2009-12-01
* Continuing r12485-12486 (cleaning around name generation)Gravatar herbelin2009-12-01
* Include Self (Type) Foo: applying a (Type) Functor to the current contextGravatar letouzey2009-11-16
* Move Obj.magic call to the Vm moduleGravatar glondu2009-11-13
* the inlining computation at functor application was raising not_found when th...Gravatar soubiran2009-11-13
* A bit of cleaning around name generation + creation of dedicated file namegen.mlGravatar herbelin2009-11-09
* Module type expressions of the form (Fsig X) with Definition foo := bar are n...Gravatar soubiran2009-10-28
* First debug... the renaming of librairies was not working and auto/dn were no...Gravatar soubiran2009-10-23
* This big commit addresses two problems:Gravatar soubiran2009-10-21
* Removal of trailing spaces.Gravatar serpyc2009-10-04