aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/obligations.mli
Commit message (Expand)AuthorAge
* Making Proof_global terminator generic in external tactics.Gravatar Pierre-Marie Pédrot2016-09-08
* Rework treatment of default transparency of obligationsGravatar Matthieu Sozeau2016-06-27
* Moving the use of Tactic_option from Obligations to G_obligations.Gravatar Pierre-Marie Pédrot2016-03-19
* Implement support for universe binder lists in Instance and Program Fixpoint/...Gravatar Matthieu Sozeau2016-01-23
* Update copyright headers.Gravatar Maxime Dénès2016-01-20
* Allow program hooks to see the refined universe_context at the end of aGravatar Matthieu Sozeau2015-11-19
* Avoid type checking private_constants (side_eff) again during Qed (#4357).Gravatar Enrico Tassi2015-10-28
* Removing dead code.Gravatar Pierre-Marie Pédrot2015-02-02
* Add the possibility of defining opaque terms with program.Gravatar mlasson2015-01-21
* Update headers.Gravatar Maxime Dénès2015-01-12
* Proofs now take and return an evar_universe_context, simplifying interfacesGravatar Matthieu Sozeau2014-06-18
* Moving hook code from Future to Lemmas. This seemed to disrupt compilation ofGravatar Pierre-Marie Pédrot2014-06-08
* This commit adds full universe polymorphism and fast projections to Coq.Gravatar Matthieu Sozeau2014-05-06
* Remove many superfluous 'open' indicated by ocamlc -w +33Gravatar Pierre Letouzey2014-03-05
* Removing useless meta-related functions.Gravatar Pierre-Marie Pédrot2013-12-03
* Makes the new Proofview.tactic the basic type of Ltac.Gravatar aspiwack2013-11-02
* At least made the evar type opaque! There are still 5 remaining unsafeGravatar ppedrot2013-09-18
* get rid of closures in global/proof stateGravatar gareuselesinge2013-08-08
* State Transaction MachineGravatar gareuselesinge2013-08-08
* Allowing (Co)Fixpoint to be defined local and Let-style.Gravatar ppedrot2013-03-11
* Modulification of identifierGravatar ppedrot2012-12-14
* Moved Intset and Intmap to Int namespace.Gravatar ppedrot2012-12-14
* Updating headers.Gravatar herbelin2012-08-08
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* Getting rid of Pp.msgnl and Pp.message.Gravatar ppedrot2012-06-01
* global_reference migrated from Libnames to new Globnames, less deps in gramma...Gravatar letouzey2012-05-29
* New files intf/constrexpr.mli and intf/notation_term.mli out of TopconstrGravatar letouzey2012-05-29
* Evar_kinds.mli containing former Evd.hole_kind, avoid deps on EvdGravatar letouzey2012-05-29
* Fix bugs related to Program integration.Gravatar msozeau2012-03-19
* Fix merge and add missing file.Gravatar msozeau2012-03-14
* Final part of moving Program code inside the main code. Adapted add_definitio...Gravatar msozeau2012-03-14