aboutsummaryrefslogtreecommitdiffhomepage
path: root/vernac/obligations.ml
Commit message (Expand)AuthorAge
* Correct some spelling errorsmasterGravatar Benjamin Barenblat2018-07-22
* Change QuestionMark for better record field missing error message.Gravatar Siddharth Bhat2018-07-17
* Swapping Context and Constr: defining declarations on constr in Constr.Gravatar Hugo Herbelin2018-06-27
* Merge PR #7906: universes_of_constr don't include universes of monomorphic co...Gravatar Pierre-Marie Pédrot2018-06-26
|\
| * universes_of_constr don't include universes of monomorphic constantsGravatar Gaëtan Gilbert2018-06-26
* | Fix handling of universe context for expanded program obligations.Gravatar Matthieu Sozeau2018-06-22
|/
* [api] Misctypes removal: miscellaneous aliases.Gravatar Emilio Jesus Gallego Arias2018-06-12
* Merge PR #7114: Fix #7113: Program Let Fixpoint in section causes anomalyGravatar Matthieu Sozeau2018-06-04
|\
* \ Merge PR #7349: Fix an anomaly when calling Obligation 0 or Obligation -1.Gravatar Matthieu Sozeau2018-06-04
|\ \
* | | [api] Move `Constrexpr` to the `interp` module.Gravatar Emilio Jesus Gallego Arias2018-05-31
* | | Merge PR #7558: [api] Make `vernac/` self-contained.Gravatar Maxime Dénès2018-05-30
|\ \ \
| | | * Fix #7113: Program Let Fixpoint in section causes anomalyGravatar Gaëtan Gilbert2018-05-30
| |_|/ |/| |
| * | [tactics] Turn boolean locality hint parameter into a named one.Gravatar Emilio Jesus Gallego Arias2018-05-27
* | | Remove some occurrences of Evd.emptyGravatar Maxime Dénès2018-05-25
|/ /
* | [api] Move `opacity_flag` to `Proof_global`.Gravatar Emilio Jesus Gallego Arias2018-05-23
| * Fix an anomaly when calling Obligation 0 or Obligation -1.Gravatar Théo Zimmermann2018-05-21
* | Split off Universes functions about substitutions and constraintsGravatar Gaëtan Gilbert2018-05-17
* | Split off Universes functions dealing with generating new universes.Gravatar Gaëtan Gilbert2018-05-17
* | Split off Universes functions dealing with names.Gravatar Gaëtan Gilbert2018-05-17
|/
* [api] Rename `global_reference` to `GlobRef.t` to follow kernel style.Gravatar Emilio Jesus Gallego Arias2018-05-04
* Evar maps contain econstrs.Gravatar Gaëtan Gilbert2018-04-13
* Allow using cumulativity without forcing strict constraints.Gravatar Gaëtan Gilbert2018-03-09
* Deprecate UState aliases in Evd.Gravatar Gaëtan Gilbert2018-03-06
* [econstr] Continue consolidation of EConstr API under `interp`.Gravatar Emilio Jesus Gallego Arias2018-02-28
* [ast] Improve precision of Ast location recognition in serialization.Gravatar Emilio Jesus Gallego Arias2018-02-22
* [flags] Make program_mode a parameter for commands in vernac.Gravatar Emilio Jesus Gallego Arias2017-12-17
* Merge PR #6275: [summary] Allow typed projections from global state.Gravatar Maxime Dénès2017-12-12
|\
| * [summary] Adapt STM to the new Summary API.Gravatar Emilio Jesus Gallego Arias2017-12-09
* | Fix #6323: stronger restrict universe context vs abstract.Gravatar Gaëtan Gilbert2017-12-06
|/
* Cleanup API for registering universe binders.Gravatar Matthieu Sozeau2017-12-01
* Merge PR #1033: Universe binder improvementsGravatar Maxime Dénès2017-11-28
|\
* | [api] Remove aliases of `Evar.t`Gravatar Emilio Jesus Gallego Arias2017-11-26
| * Restrict universe context when declaring constants in obligations.Gravatar Gaëtan Gilbert2017-11-25
| * Fix obligations handling of universes anticipating stronger restrictGravatar Matthieu Sozeau2017-11-25
| * Use Entries.constant_universes_entry more.Gravatar Gaëtan Gilbert2017-11-24
| * When declaring constants/inductives use ContextSet if monomorphic.Gravatar Gaëtan Gilbert2017-11-24
| * Stop exposing UState.universe_context and its Evd wrapper.Gravatar Gaëtan Gilbert2017-11-24
| * Separate checking univ_decls and obtaining universe binder names.Gravatar Gaëtan Gilbert2017-11-24
| * Use Maps and ids for universe bindersGravatar Gaëtan Gilbert2017-11-24
|/
* Fix universe polymorphic Program obligations.Gravatar Matthieu Sozeau2017-11-22
* [api] Insert miscellaneous API deprecation back to core.Gravatar Emilio Jesus Gallego Arias2017-11-13
* [api] Another large deprecation, `Nameops`Gravatar Emilio Jesus Gallego Arias2017-11-13
* [api] Move structures deprecated in the API to the core.Gravatar Emilio Jesus Gallego Arias2017-11-06
* Merge PR #1120: Fixing BZ#5762 (supporting implicit arguments in "where" clau...Gravatar Maxime Dénès2017-10-20
|\
| * Fixing #5762 (supporting imp. args. in "where" clause of an inductive def.).Gravatar Hugo Herbelin2017-10-05
* | [vernac] Remove `Qed exporting` syntax.Gravatar Emilio Jesus Gallego Arias2017-09-29
|/
* Don't lose names in UState.universe_context.Gravatar Gaëtan Gilbert2017-09-19
* Allow declaring universe constraints at definition level.Gravatar Matthieu Sozeau2017-09-19
* Merge PR #841: Timorous fix of bug #5598 on global existing class in sectionsGravatar Maxime Dénès2017-08-16
|\
* | Statically ensuring that inlined entries out of the kernel have no effects.Gravatar Pierre-Marie Pédrot2017-07-26