aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
Commit message (Expand)AuthorAge
* Type-safe Egramml.grammar_prod_item.Gravatar Pierre-Marie Pédrot2015-10-27
* Finer type for Pcoq.interp_entry_name.Gravatar Pierre-Marie Pédrot2015-10-27
* Indexing existentially quantified entries returned by interp_entry_name.Gravatar Pierre-Marie Pédrot2015-10-27
* Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-26
|\
| * Minor module cleanup : error HigherOrderInclude was never happeningGravatar Pierre Letouzey2015-10-25
* | Pcoq.prod_entry_key now uses a GADT to statically enforce typedness.Gravatar Pierre-Marie Pédrot2015-10-21
* | Boxing the Goal.enter primitive into a record type.Gravatar Pierre-Marie Pédrot2015-10-20
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-19
|\|
* | Constraining refine to monotonic functions.Gravatar Pierre-Marie Pédrot2015-10-18
| * Miscellaneous typos, spacing, US spelling in comments or variable names.Gravatar Hugo Herbelin2015-10-18
* | Clarifying and documenting the UState API.Gravatar Pierre-Marie Pédrot2015-10-17
| * Lemmas accept the Local flag.Gravatar Pierre-Marie Pédrot2015-10-17
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-15
|\|
| * Remove -vm flag of coqtop.Gravatar Maxime Dénès2015-10-14
| * Fixing bug #4367: Wrong error message in unification.Gravatar Pierre-Marie Pédrot2015-10-14
| * Fix some typos.Gravatar Guillaume Melquiond2015-10-13
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-12
|\|
| * Fix Definition id := Eval <redexpr> in by passing the right universeGravatar Matthieu Sozeau2015-10-12
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-10
|\|
| * Code cleaning in VM (with Benjamin).Gravatar Maxime Dénès2015-10-09
| * Fix Next Obligation to not raise an anomaly in case of mutualGravatar Matthieu Sozeau2015-10-09
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-09
|\|
| * Axioms now support the universe binding syntax.Gravatar Pierre-Marie Pédrot2015-10-08
| * aux_file: export API to ease writing of a Proof Using annotator.Gravatar Enrico Tassi2015-10-08
| * Proof using: let-in policy, optional auto-clear, forward closure*Gravatar Enrico Tassi2015-10-08
| * Spawn: use each socket exclusively for writing or readingGravatar Enrico Tassi2015-10-08
| * Goptions: new value type: optional stringGravatar Enrico Tassi2015-10-08
| * Univs: fix FingerTree contrib.Gravatar Matthieu Sozeau2015-10-07
| * Univs: add Strict Universe Declaration option (on by default)Gravatar Matthieu Sozeau2015-10-07
* | Splitting kernel universe code in two modules.Gravatar Pierre-Marie Pédrot2015-10-06
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-06
|\|
| * Univs: fix handling of evar_map in identity coercion construction.Gravatar Matthieu Sozeau2015-10-05
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-02
|\|
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-10-02
|\ \
| | * Fix after rebase...Gravatar Matthieu Sozeau2015-10-02
| | * Univs: fix inference of the lowest sort for records.Gravatar Matthieu Sozeau2015-10-02
| | * Univs: correcly compute the levels of records when they fall in Prop.Gravatar Matthieu Sozeau2015-10-02
| | * Univs/program: handle side effects in obligations.Gravatar Matthieu Sozeau2015-10-02
| | * Univs: fix Show Universes.Gravatar Matthieu Sozeau2015-10-02
| | * Univs: fix environment handling in scheme building.Gravatar Matthieu Sozeau2015-10-02
| | * Univs: fix after rebase (from_ctx/from_env)Gravatar Matthieu Sozeau2015-10-02
| | * Univs: fix many evar_map initializations and leaks.Gravatar Matthieu Sozeau2015-10-02
| | * Universes: enforce Set <= i for all Type occurrences.Gravatar Matthieu Sozeau2015-10-02
| |/
| * Prevent States.intern_state and System.extern_intern from looking up files in...Gravatar Guillaume Melquiond2015-09-29
| * Remove some uses of Loadpath.get_paths.Gravatar Guillaume Melquiond2015-09-29
| * Make -load-vernac-object respect the loadpath.Gravatar Guillaume Melquiond2015-09-28
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-09-25
|\|
| * The -require option now accepts a logical path instead of a physical one.Gravatar Pierre-Marie Pédrot2015-09-25
| * Updating the documentation and the toolchain w.r.t. the change in -compile.Gravatar Pierre-Marie Pédrot2015-09-25
| * The -compile option now accepts ".v" files and outputs a warning otherwise.Gravatar Pierre-Marie Pédrot2015-09-25