aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing
Commit message (Expand)AuthorAge
* - Add modulo_delta_types flag for unification to allow fullGravatar msozeau2011-03-13
* Reverted commit r13893 about propagation of more informativeGravatar herbelin2011-03-07
* Added propagation of evars unification failure reasons for betterGravatar herbelin2011-03-07
* Forgotten removal of ',' in 'fun' rule: it has to come with the lambda notationGravatar herbelin2011-03-05
* - Fix treatment of globality flag for typeclass instance hints (theyGravatar msozeau2011-02-14
* Annotations at functor applications:Gravatar letouzey2011-02-11
* A fine-grain control of inlining at functor application via priority levelsGravatar letouzey2011-01-31
* Remove the "Boxed" syntaxes and the const_entry_boxed fieldGravatar letouzey2011-01-28
* Fix compilation with camlp5 (Closes: #2487)Gravatar glondu2011-01-25
* Add "Print Sorted Universes"Gravatar glondu2011-01-11
* ARGUMENT EXTEND: forbid TYPED simultaneously with {RAW,GLOB}_TYPEDGravatar glondu2010-12-25
* Avoid "open {Pcoq,Extrawit}" clauses in expansion of EXTEND commandsGravatar glondu2010-12-25
* More {raw => glob} changes for consistencyGravatar glondu2010-12-24
* Remove obsolete script univdot, update dev doc about universesGravatar glondu2010-12-24
* Rename rawterm.ml into glob_term.mlGravatar glondu2010-12-23
* Change of nomenclature: rawconstr -> glob_constrGravatar glondu2010-12-23
* Don't interpret VMcast as an ordinary type cast in Definition a := t <: T.Gravatar herbelin2010-12-09
* SearchAbout: who has never been annoyed by the [ ] syntax ?Gravatar letouzey2010-11-19
* adapt slighlty r13642 to support both camlp4 and camlp5-5 and camlp5-6Gravatar letouzey2010-11-18
* Support for camlp5 6.02.0 (Closes: #2432)Gravatar glondu2010-11-16
* About "unsupported" unicode characters in notations.Gravatar herbelin2010-10-17
* Backporting r13521 from branch 8.3 to trunk (fixing bug #2406, loopingGravatar herbelin2010-10-11
* Export the "bullet" grammar entryGravatar glondu2010-10-08
* Remove Explain* vernacsGravatar glondu2010-10-06
* Remove VernacGoGravatar glondu2010-10-06
* Added multiple implicit arguments rules per name.Gravatar herbelin2010-10-03
* Making display of various informations about constants more modular:Gravatar herbelin2010-10-03
* Fixed a little printing bug with "About" on an undefined constant.Gravatar herbelin2010-10-03
* Simplify tactic(_)-bound arguments in TACTIC EXTEND rulesGravatar glondu2010-09-30
* Remove some occurrences of "open Termops"Gravatar glondu2010-09-28
* Some dead code removal, thanks to Oug analyzerGravatar letouzey2010-09-24
* Improved printing of Unfoldable constants in hints databases (usedGravatar herbelin2010-09-02
* r13359 continued: removed native treatment for λ (lambda) and Π (Pi)Gravatar herbelin2010-07-30
* Rather quick hack to make basic unicode notations available byGravatar herbelin2010-07-29
* Updated all headers for 8.3 and trunkGravatar herbelin2010-07-24
* Extension of the recursive notations mechanismGravatar herbelin2010-07-22
* Constrintern: unified push_name_env and push_loc_name_env; madeGravatar herbelin2010-07-22
* Cleaned a bit the grammar and terminology for binders (see dev/doc/changes.txt).Gravatar herbelin2010-07-22
* Fixed parsing of "Generalizable Variable A" ("Variable" turns to be a keyword).Gravatar herbelin2010-07-18
* Finish adding out-of-the-box support for camlp4Gravatar letouzey2010-07-09
* Applying François' patches about Canonical Projections (see #2302 and #2334).Gravatar herbelin2010-06-26
* New script dev/tools/change-header to automatically update Coq files headers.Gravatar herbelin2010-06-22
* Fixing spelling: pr_coma -> pr_commaGravatar herbelin2010-06-12
* Using vernac parsing for FunctionGravatar jforest2010-06-08
* Added support for Ltac-matching terms with variables bound in the patternGravatar herbelin2010-06-06
* A new command Compute foo, shortcut for Eval vm_compute in fooGravatar letouzey2010-06-04
* Added command "Locate Ltac qid".Gravatar herbelin2010-06-03
* deporting Coq specific code from ide to toplevel.Gravatar vgross2010-05-31
* Add (almost) compatibility with camlp4, without breaking support for camlp5Gravatar letouzey2010-05-19
* Nicer representation of tokens, more independant of camlp*Gravatar letouzey2010-05-19