aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/command.ml
Commit message (Expand)AuthorAge
* Fix handling of anonymous Type in template universe polymorphic inductivesGravatar Matthieu Sozeau2014-06-04
* - Fix treatment of global universe constraints which should be passed alongGravatar Matthieu Sozeau2014-05-06
* Proper calculation of constructor levels, forgetting the level of lets.Gravatar Matthieu Sozeau2014-05-06
* Retype application of fix_proto to get the right universes in ProgramGravatar Matthieu Sozeau2014-05-06
* Fix restrict_universe_context removing some universes that do appear in the t...Gravatar Matthieu Sozeau2014-05-06
* Fix declarations of monomorphic assumptionsGravatar Matthieu Sozeau2014-05-06
* Fix program Fixpoint not taking care of universes.Gravatar Matthieu Sozeau2014-05-06
* - Fix bug preventing apply from unfolding Fixpoints.Gravatar Matthieu Sozeau2014-05-06
* Adapt Y. Bertot's path on private inductives (now the keyword is "Private").Gravatar Yves Bertot2014-05-06
* Correct rebase on STM code. Thanks to E. Tassi for help on dealing withGravatar Matthieu Sozeau2014-05-06
* Rework handling of universes on top of the STM, allowing for delayedGravatar Matthieu Sozeau2014-05-06
* This commit adds full universe polymorphism and fast projections to Coq.Gravatar Matthieu Sozeau2014-05-06
* Removing Autoinstance once and for all.Gravatar Pierre-Marie Pédrot2014-04-25
* Remove some dead-code (thanks to ocaml warnings)Gravatar Pierre Letouzey2014-03-05
* Useless Evd.create_evar_defs.Gravatar Pierre-Marie Pédrot2013-12-30
* STM: capture type checking error (Closes: 3195)Gravatar Enrico Tassi2013-12-24
* Qed: feedback when type checking is doneGravatar Enrico Tassi2013-12-24
* Adding generic solvers to term holes. For now, no resolution mechanism norGravatar Pierre-Marie Pédrot2013-11-27
* Fixup bug 3145Gravatar pboutill2013-11-03
* Makes the new Proofview.tactic the basic type of Ltac.Gravatar aspiwack2013-11-02
* Future: better doc + restore ~pure optimizationGravatar gareuselesinge2013-10-31
* Conv_orable made functional and part of pre_envGravatar gareuselesinge2013-10-31
* More monomorphic List.mem + List.assoc + ...Gravatar letouzey2013-10-24
* Turn many List.assoc into List.assoc_fGravatar letouzey2013-10-24
* cList: set-as-list functions are now with an explicit comparisonGravatar letouzey2013-10-23
* declaration_hooks use EphemeronGravatar gareuselesinge2013-10-18
* Future: ported to Ephemeron + exception enhancingGravatar gareuselesinge2013-10-18
* Removing a bunch of generic equalities.Gravatar ppedrot2013-09-27
* Removing almost all new_untyped_evar, and a bunch of Evd.add.Gravatar ppedrot2013-09-18
* get rid of closures in global/proof stateGravatar gareuselesinge2013-08-08
* State Transaction MachineGravatar gareuselesinge2013-08-08
* Use the Hook module here and there.Gravatar ppedrot2013-05-12
* Use definition_entry to declare local definitionsGravatar gareuselesinge2013-05-09
* A uniformization step around understand_* and interp_* functions.Gravatar herbelin2013-05-09
* Uniformization: isevars -> evdref/sigma/evdGravatar herbelin2013-05-09
* Fixing r16487 on sharing evars between multiple parameters (missing List.rev).Gravatar herbelin2013-05-09
* Uniformizing the [if_warn] flag used for warning printing and putGravatar ppedrot2013-05-08
* Declaration of multiple hypotheses or parameters now share typingGravatar herbelin2013-05-08
* Share more information between constructors and arity of an inductiveGravatar herbelin2013-05-08
* Merging Context and Sign.Gravatar ppedrot2013-04-29
* Splitting Term into five unrelated interfaces:Gravatar ppedrot2013-04-29
* Fix bug# 2994, 2971 about better error messages.Gravatar msozeau2013-03-22
* Making local variable warning verbose by default.Gravatar ppedrot2013-03-18
* Modules and ppvernac, sequel of Enrico's commit 16261Gravatar letouzey2013-03-13
* Restrict (try...with...) to avoid catching critical exn (part 13)Gravatar 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
* Uniformization of the "anomaly" command.Gravatar ppedrot2013-01-28
* New implementation of the conversion test, using normalization by evaluation toGravatar mdenes2013-01-22
* Modulification of identifierGravatar ppedrot2012-12-14