aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing/g_vernac.ml4
Commit message (Expand)AuthorAge
* Adding generic solvers to term holes. For now, no resolution mechanism norGravatar Pierre-Marie Pédrot2013-11-27
* Fixes parsing of all: followed by a typechecking/evaluation command.Gravatar aspiwack2013-11-02
* New option Default Goal Selector.Gravatar aspiwack2013-11-02
* Adds a new goal selector "all:".Gravatar aspiwack2013-11-02
* STM: add "Stm Wait" to wait for the slaves to complete their jobsGravatar gareuselesinge2013-10-10
* STM: new command "Stm PrintDag" to force printing the dag to /tmpGravatar gareuselesinge2013-10-07
* Modulification and removing of structural equality in Stateid.Gravatar ppedrot2013-08-19
* Support Proof GeneralGravatar gareuselesinge2013-08-08
* State Transaction MachineGravatar gareuselesinge2013-08-08
* Added a Print Debug GC command that displays the current state ofGravatar ppedrot2013-08-01
* Granting bug #3098: adding priority to Existing Instances.Gravatar ppedrot2013-08-01
* More dynamic argument scopesGravatar letouzey2013-07-17
* Added a Register Inline command for the native compiler. Will be ported to th...Gravatar mdenes2013-07-10
* Fixing warning of deprecated Argument Scopes.Gravatar ppedrot2013-05-28
* Renaming SearchAbout into Search and Search into SearchHead.Gravatar herbelin2013-04-17
* More functional implementation of locality_flag and program_modeGravatar gareuselesinge2013-04-15
* Modules and ppvernac, sequel of Enrico's commit 16261Gravatar letouzey2013-03-13
* Allowing (Co)Fixpoint to be defined local and Let-style.Gravatar ppedrot2013-03-11
* Added a Local Definition vernacular command. This type of definitionGravatar ppedrot2013-03-11
* Useless use of hooks in VernacDefinition. In addition, this wasGravatar ppedrot2013-02-10
* New implementation of the conversion test, using normalization by evaluation toGravatar mdenes2013-01-22
* Monomorphization (parsing)Gravatar ppedrot2012-11-25
* Fixed #2926:Gravatar ppedrot2012-10-29
* Moved Compat to parsing. This permits to break the dependency of theGravatar ppedrot2012-10-04
* Remove some more "open" and dead code thanks to OCaml4 warningsGravatar letouzey2012-10-02
* Added support for option Local (at module level) in Tactic Notation.Gravatar herbelin2012-08-11
* Updating headers.Gravatar herbelin2012-08-08
* Re-allow Reset in compiled filesGravatar letouzey2012-07-11
* A prototype implementation of a Print Namespace command.Gravatar aspiwack2012-07-06
* Notation: a new annotation "compat 8.x" extending "only parsing"Gravatar letouzey2012-07-05
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* Added a color output to Coqtop.Gravatar ppedrot2012-06-04
* global_reference migrated from Libnames to new Globnames, less deps in gramma...Gravatar letouzey2012-05-29
* Basic stuff about constr_expr migrated from topconstr to constrexpr_opsGravatar letouzey2012-05-29
* Migrate the grammar entry about "Ltac" into g_vernac.ml4.Gravatar letouzey2012-05-29
* New files intf/constrexpr.mli and intf/notation_term.mli out of TopconstrGravatar letouzey2012-05-29
* Glob_term now mli-only, operations now in Glob_opsGravatar letouzey2012-05-29
* locus.mli for occurrences+clauses, misctypes.mli for various little thingsGravatar letouzey2012-05-29
* Vernacexpr is now a mli-only file, locality stuff now in locality.mlGravatar letouzey2012-05-29
* Program: avoid staying in program mode after a failed Program commandGravatar letouzey2012-04-26
* Slight change in the semantics of arguments scopes: scopes can noGravatar herbelin2012-03-26
* Remove undocumented command "Delete foo"Gravatar letouzey2012-03-23
* Final part of moving Program code inside the main code. Adapted add_definitio...Gravatar msozeau2012-03-14
* Noise for nothingGravatar pboutill2012-03-02
* Arguments supports extra notation scopesGravatar gareuselesinge2012-02-14
* Fix camlp4 compilationGravatar pboutill2012-01-31
* Added an pattern / occurence syntax for vm_compute.Gravatar ppedrot2012-01-30
* Removed a seemingly unused argument in Require of modules, introduced 10 year...Gravatar ppedrot2012-01-23
* Reverted previous commit, which broke library compilation.Gravatar ppedrot2012-01-20
* This is a quick hack to permit the parsing of the locality flag in the Progra...Gravatar ppedrot2012-01-20