aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing
Commit message (Expand)AuthorAge
...
* | Change default for notations with variables bound to both terms and binders.Gravatar Hugo Herbelin2018-02-20
* | Notations: Adding modifiers to tell which kind of binder a constr can parse.Gravatar Hugo Herbelin2018-02-20
* | Notations: A step in cleaning constr_entry_key.Gravatar Hugo Herbelin2018-02-20
* | Moving Metasyntax.register_grammar to Pcoq for usability in Egramcoq.Gravatar Hugo Herbelin2018-02-20
* | Adding support for parsing subterms of a notation as "pattern".Gravatar Hugo Herbelin2018-02-20
* | Adding patterns in the category of binders for notations.Gravatar Hugo Herbelin2018-02-20
* | Renaming binders into binderlists in egramcoq.ml.Gravatar Hugo Herbelin2018-02-20
* | Introducing an intermediary type "constr_prod_entry_key" for grammar producti...Gravatar Hugo Herbelin2018-02-20
* | Rephrasing ETBinderList with a self-documenting and invariant-carrying argument.Gravatar Hugo Herbelin2018-02-20
|/
* Change references to CAMLP4 to CAMLP5 to be more accurate since we noGravatar Jim Fehrle2018-02-17
* [vernac] Mutual theorems (VernacStartTheoremProof) always have namesGravatar Vincent Laporte2018-02-01
* [vernac] Remove VernacGoal, allow anonymous definitions in VernacDefinitionGravatar Vincent Laporte2018-02-01
* [vernac] vernac_expr no longer recursiveGravatar Vincent Laporte2018-01-08
* Merge PR #6433: [flags] Move global time flag into an attribute.Gravatar Maxime Dénès2017-12-29
|\
* | [api] Also deprecate constructors of Decl_kinds.Gravatar Emilio Jesus Gallego Arias2017-12-23
| * [flags] Move global time flag into an attribute.Gravatar Emilio Jesus Gallego Arias2017-12-23
|/
* Separate vernac controls and regular commands.Gravatar Maxime Dénès2017-12-20
* Merge PR #978: In printing, experimenting factorizing "match" clauses with sa...Gravatar Maxime Dénès2017-12-14
|\
| * Removing cumbersome location in multiple patterns.Gravatar Hugo Herbelin2017-12-12
* | [summary] Allow typed projections from global state + rework of internals.Gravatar Emilio Jesus Gallego Arias2017-12-09
|/
* Proper nametab handling of global universe namesGravatar Matthieu Sozeau2017-12-01
* Remove "obsolete_locality" and fix STM vernac classification.Gravatar Maxime Dénès2017-11-29
* Merge PR #6253: Fixing inconsistent associativity of level 10 in the table of...Gravatar Maxime Dénès2017-11-29
|\
| * A cosmetic standardization: adding a space in g_constr.ml4.Gravatar Hugo Herbelin2017-11-27
| * Releasing level "11" of "pattern".Gravatar Hugo Herbelin2017-11-27
| * Fixing associativity registered for level 10.Gravatar Hugo Herbelin2017-11-27
* | Allow local universe renaming in Print.Gravatar Gaëtan Gilbert2017-11-25
|/
* Merge PR #6167: Fixing factorization of recursive notations with an atomic se...Gravatar Maxime Dénès2017-11-23
|\
* \ Merge PR #6200: Remove pidentref grammar entry.Gravatar Maxime Dénès2017-11-23
|\ \
| | * Fixing factorization of recursive notations in the case of an atomic separator.Gravatar Hugo Herbelin2017-11-20
| * | Remove pidentref grammar entry.Gravatar Gaëtan Gilbert2017-11-20
| |/
* / [parser] Remove unnecessary statically initialized hook.Gravatar Emilio Jesus Gallego Arias2017-11-19
|/
* Fix FIXME: use OCaml 4.02 generative functors when available.Gravatar Gaëtan Gilbert2017-11-01
* Parse [Proof using Type] without translating Type to an id.Gravatar Gaëtan Gilbert2017-10-10
* [vernac] Remove "Proof using" hacks from parser.Gravatar Emilio Jesus Gallego Arias2017-10-10
* Merge PR #1114: Generic handling of nameable objects for pluginsGravatar Maxime Dénès2017-10-09
|\
* \ Merge PR #1119: Fixing bug BZ#5769 (generating a name "_" out of a type "_som...Gravatar Maxime Dénès2017-10-06
|\ \
| * | Distinguishing pseudo-letters out of the set of unicode letters.Gravatar Hugo Herbelin2017-10-05
| | * Implementing a generic mechanism for locating named objects from Coq side.Gravatar Pierre-Marie Pédrot2017-10-03
| |/ |/|
* | Merge PR #1094: Fixing a little parsing bug with level 90 introduced in 3e70e...Gravatar Maxime Dénès2017-10-03
|\ \
* \ \ Merge PR #1040: Efficient fresh name generationGravatar Maxime Dénès2017-10-03
|\ \ \
* | | | [vernac] Remove `Qed exporting` syntax.Gravatar Emilio Jesus Gallego Arias2017-09-29
| |_|/ |/| |
| * | Efficient fresh name generation relying on sets.Gravatar Pierre-Marie Pédrot2017-09-28
|/ /
* | Merge PR #688: Binding universe constraints in Definition/Inductive/etc...Gravatar Maxime Dénès2017-09-26
|\ \
| | * Fixing a little parsing bug with level 90 introduced in 3e70ea9c.Gravatar Hugo Herbelin2017-09-25
| |/ |/|
* | Remove STM vernaculars.Gravatar Maxime Dénès2017-09-19
| * Allow declaring universe binders with no constraints with @{|}Gravatar Gaëtan Gilbert2017-09-19
| * Allow declaring universe constraints at definition level.Gravatar Matthieu Sozeau2017-09-19
| * Allow empty instance parsing @{}Gravatar Matthieu Sozeau2017-09-19
|/
* Merge PR #939: [general] Merge parsing with highparsing, put toplevel at the ...Gravatar Maxime Dénès2017-09-15
|\