aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/command.ml
Commit message (Expand)AuthorAge
...
* 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
* Moved Intset and Intmap to Int namespace.Gravatar ppedrot2012-12-14
* Implemented a full-fledged equality on [constr_expr]. By the way,Gravatar ppedrot2012-12-14
* Monomorphization (toplevel)Gravatar ppedrot2012-11-26
* Monomorphized a lot of equalities over OCaml integers, thanks toGravatar ppedrot2012-11-08
* Remove some more "open" and dead code thanks to OCaml4 warningsGravatar letouzey2012-10-02
* Cleaning interface of Util.Gravatar ppedrot2012-09-18
* Some documentation and cleaning of CList and Util interfaces.Gravatar ppedrot2012-09-15
* Moving Utils.list_* to a proper CList module, which includes stdlibGravatar ppedrot2012-09-14
* The new ocaml compiler (4.00) has a lot of very cool warnings,Gravatar regisgia2012-09-14
* Fix computation of obligations for mutually recursive definitions.Gravatar msozeau2012-09-06
* Assumption commands are now displayed as unsafe in Coqide.Gravatar aspiwack2012-08-24
* Updating headers.Gravatar herbelin2012-08-08
* Bug 2838: ExplApp in mutual inductive parametersGravatar pboutill2012-07-12
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* Fixing previous commit (something strange happened...)Gravatar ppedrot2012-06-04
* Replacing some str with strbrkGravatar ppedrot2012-06-04
* Separated notice vs info messages, and cleaned up the interface a bit.Gravatar ppedrot2012-06-04
* Forward-port fixes from 8.4 (15358, 15353, 15333).Gravatar msozeau2012-06-04
* Cleaning Pp.ppnl useGravatar ppedrot2012-06-01
* More uniformisation in Pp.warn functions.Gravatar ppedrot2012-05-30
* global_reference migrated from Libnames to new Globnames, less deps in gramma...Gravatar letouzey2012-05-29
* Basic stuff about constr_expr migrated from topconstr to constrexpr_opsGravatar letouzey2012-05-29
* New files intf/constrexpr.mli and intf/notation_term.mli out of TopconstrGravatar letouzey2012-05-29
* locus.mli for occurrences+clauses, misctypes.mli for various little thingsGravatar letouzey2012-05-29
* Evar_kinds.mli containing former Evd.hole_kind, avoid deps on EvdGravatar letouzey2012-05-29
* Implicit arguments of Definition are taken from the type when given by the user.Gravatar pboutill2012-04-27
* Bug 2733 : { } implicits and FixpointsGravatar pboutill2012-04-17
* Fix interface of resolve_typeclasses: onlyargs -> with_goals:Gravatar msozeau2012-03-20
* Continuing r15045-15046 and r15055 (fixing bug #2732 about atomicGravatar herbelin2012-03-20
* Fix bugs related to Program integration.Gravatar msozeau2012-03-19
* Final part of moving Program code inside the main code. Adapted add_definitio...Gravatar msozeau2012-03-14
* Integrated obligations/eterm and program well-founded fixpoint building to to...Gravatar msozeau2012-03-14
* Noise for nothingGravatar pboutill2012-03-02
* A pass on warning printings. Made systematic the use of msg_warning soGravatar herbelin2011-12-17
* Proof using ...Gravatar gareuselesinge2011-12-12
* Merge subinstances branch by me and Tom Prince.Gravatar msozeau2011-11-17
* Various simplifications about constant_of_delta and mind_of_deltaGravatar letouzey2011-10-11
* Revert "Add [Polymorphic] flag for defs"Gravatar msozeau2011-04-13
* Add [Polymorphic] flag for defsGravatar msozeau2011-04-13