aboutsummaryrefslogtreecommitdiff
path: root/toplevel/command.ml
AgeCommit message (Expand)Author
2013-03-13Restrict (try...with...) to avoid catching critical exn (part 13)letouzey
2013-03-11Allowing (Co)Fixpoint to be defined local and Let-style.ppedrot
2013-03-11Added a Local Definition vernacular command. This type of definitionppedrot
2013-01-28Uniformization of the "anomaly" command.ppedrot
2013-01-22New implementation of the conversion test, using normalization by evaluation tomdenes
2012-12-14Modulification of identifierppedrot
2012-12-14Moved Intset and Intmap to Int namespace.ppedrot
2012-12-14Implemented a full-fledged equality on [constr_expr]. By the way,ppedrot
2012-11-26Monomorphization (toplevel)ppedrot
2012-11-08Monomorphized a lot of equalities over OCaml integers, thanks toppedrot
2012-10-02Remove some more "open" and dead code thanks to OCaml4 warningsletouzey
2012-09-18Cleaning interface of Util.ppedrot
2012-09-15Some documentation and cleaning of CList and Util interfaces.ppedrot
2012-09-14Moving Utils.list_* to a proper CList module, which includes stdlibppedrot
2012-09-14The new ocaml compiler (4.00) has a lot of very cool warnings,regisgia
2012-09-06Fix computation of obligations for mutually recursive definitions.msozeau
2012-08-24Assumption commands are now displayed as unsafe in Coqide.aspiwack
2012-08-08Updating headers.herbelin
2012-07-12Bug 2838: ExplApp in mutual inductive parameterspboutill
2012-06-22Added an indirection with respect to Loc in Compat. As many [open Compat]ppedrot
2012-06-04Fixing previous commit (something strange happened...)ppedrot
2012-06-04Replacing some str with strbrkppedrot
2012-06-04Separated notice vs info messages, and cleaned up the interface a bit.ppedrot
2012-06-04Forward-port fixes from 8.4 (15358, 15353, 15333).msozeau
2012-06-01Cleaning Pp.ppnl useppedrot
2012-05-30More uniformisation in Pp.warn functions.ppedrot
2012-05-29global_reference migrated from Libnames to new Globnames, less deps in gramma...letouzey
2012-05-29Basic stuff about constr_expr migrated from topconstr to constrexpr_opsletouzey
2012-05-29New files intf/constrexpr.mli and intf/notation_term.mli out of Topconstrletouzey
2012-05-29locus.mli for occurrences+clauses, misctypes.mli for various little thingsletouzey
2012-05-29Evar_kinds.mli containing former Evd.hole_kind, avoid deps on Evdletouzey
2012-04-27Implicit arguments of Definition are taken from the type when given by the user.pboutill
2012-04-17Bug 2733 : { } implicits and Fixpointspboutill
2012-03-20Fix interface of resolve_typeclasses: onlyargs -> with_goals:msozeau
2012-03-20Continuing r15045-15046 and r15055 (fixing bug #2732 about atomicherbelin
2012-03-19Fix bugs related to Program integration.msozeau
2012-03-14Final part of moving Program code inside the main code. Adapted add_definitio...msozeau
2012-03-14Integrated obligations/eterm and program well-founded fixpoint building to to...msozeau
2012-03-02Noise for nothingpboutill
2011-12-17A pass on warning printings. Made systematic the use of msg_warning soherbelin
2011-12-12Proof using ...gareuselesinge
2011-11-17Merge subinstances branch by me and Tom Prince.msozeau
2011-10-11Various simplifications about constant_of_delta and mind_of_deltaletouzey
2011-04-13Revert "Add [Polymorphic] flag for defs"msozeau
2011-04-13Add [Polymorphic] flag for defsmsozeau
2011-02-10Fixpoints are traverse during implicits arguments search to toplevelpboutill
2011-02-10Interp a definition with the implicit arguments of its local contextpboutill
2011-01-28Remove the "Boxed" syntaxes and the const_entry_boxed fieldletouzey
2010-12-24More {raw => glob} changes for consistencyglondu
2010-12-23Rename rawterm.ml into glob_term.mlglondu