aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
...
* Goal: preventively replace an Evd.fold by an equivalent Evd.fold_undefinedGravatar letouzey2010-12-13
* Class_tactics: avoid an Evd.fold taking ages in contrib ProjectiveGeometryGravatar letouzey2010-12-13
* Avoid silent loss of data when closing an unsaved buffer.Gravatar gmelquio2010-12-13
* Sorry for the mistake in r13702Gravatar pboutill2010-12-12
* Attempt to preserve casts during a refine, especially VMcastGravatar letouzey2010-12-10
* First release of Vector library.Gravatar pboutill2010-12-10
* Don't interpret VMcast as an ordinary type cast in Definition a := t <: T.Gravatar herbelin2010-12-09
* In passing, very quick uniformization of coqdoc headers in a few files.Gravatar herbelin2010-12-09
* ZArith: for uniformity, Zdiv2 becomes Zquot2 while Zdiv2' becomes Zdiv2Gravatar letouzey2010-12-09
* Example of a simple ML tactic (Hello world).Gravatar fkirchne2010-12-09
* Fixed status of ÷ and × in coqdoc (they were seen as letter instead of symb...Gravatar herbelin2010-12-06
* Numbers and bitwise functions.Gravatar letouzey2010-12-06
* Use !Pp_control.std_ft for printing grammarsGravatar glondu2010-12-06
* Made new comm. model between coq and coqide support '-R foo ""'-style option.Gravatar herbelin2010-12-04
* Applied patch to FAQ proposed by Hendrik Tews (bug report #2446).Gravatar herbelin2010-12-04
* Fixing bug #2448 (wrongly-scoped alpha-renaming in notations).Gravatar herbelin2010-12-04
* Fixing coqdoc pretty-printing of a table in Mergesort. Incidentally,Gravatar herbelin2010-12-04
* Better fix to bug #2183 ("moduleid" internal name got exposed to usersGravatar herbelin2010-12-04
* Fixing several bugs with links to notation in coqdoc, including bug #2445:Gravatar herbelin2010-12-04
* Fixing bug using explictly declared implicit arguments in inductive arities.Gravatar herbelin2010-12-03
* Redirect stdout to stderr in -ideslaveGravatar glondu2010-12-03
* Remove dead codeGravatar glondu2010-12-03
* Fixing a bug introduced in r12304 (move of interpretation ofGravatar herbelin2010-12-02
* Document new tactics in CHANGESGravatar glondu2010-12-02
* Documentation for tactic constr_eqGravatar glondu2010-12-02
* Add tactic has_evar (#2433)Gravatar glondu2010-12-02
* Add tactic is_evar (Closes: #2433)Gravatar glondu2010-12-02
* * Kernel/Term:Gravatar regisgia2010-12-01
* * Kernel/TermGravatar regisgia2010-12-01
* * Kernel/TermGravatar regisgia2010-12-01
* Dp: minor fix suggested by Virgile PrevostoGravatar letouzey2010-11-25
* CHANGES: mention some changes in trunk since the 8.3 forkGravatar letouzey2010-11-19
* SearchAbout: who has never been annoyed by the [ ] syntax ?Gravatar letouzey2010-11-19
* CHANGES: small re-sync with the one of branch v8.3Gravatar letouzey2010-11-19
* adapt slighlty r13642 to support both camlp4 and camlp5-5 and camlp5-6Gravatar letouzey2010-11-18
* Some more revision of {P,N,Z}Arith + bitwise ops in NdigitsGravatar letouzey2010-11-18
* Do not throw an error for anonymous generalized binders as they will beGravatar msozeau2010-11-18
* NZSqrt: we define sqrt_up, a square root that rounds up instead of down as sqrtGravatar letouzey2010-11-18
* NZLog: we define log2_up, a base-2 logarithm that rounds up instead of down a...Gravatar letouzey2010-11-18
* Support for camlp5 6.02.0 (Closes: #2432)Gravatar glondu2010-11-16
* Division: avoid imposing rem as an infix keyword in Z_scope and bigZ_scope.Gravatar letouzey2010-11-16
* Remove redundant clause (and fix compatibility issue)Gravatar glondu2010-11-16
* Use full path for unknown stuff in omegaGravatar glondu2010-11-16
* Minor fixes from Gregory Malecha. A typo fixed and a better (located) Gravatar msozeau2010-11-15
* Oups, fix last commit, a missing file in a vo.itargetGravatar letouzey2010-11-10
* Integer division: quot and rem (trunc convention) in addition to div and modGravatar letouzey2010-11-10
* Refresh universes in params when generating schemes (Closes: #2429)Gravatar glondu2010-11-08
* Print universes in debugging printersGravatar glondu2010-11-08
* Delayed the evar normalization in error messages to the last minuteGravatar herbelin2010-11-07
* Improved error messages in CoqIDE:Gravatar herbelin2010-11-07