aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins
Commit message (Expand)AuthorAge
* Updating headers.Gravatar herbelin2012-08-08
* Fixup for macOS 10.8 & Ocaml 4.0Gravatar pboutill2012-08-08
* Vecnacentries.dump_global silently ignores exceptionsGravatar pboutill2012-08-06
* Try to make the use of Unix.lockf in micromega compatible with Win32Gravatar letouzey2012-08-06
* Dump references in ExtractionGravatar pboutill2012-08-05
* Dump referencesGravatar pboutill2012-08-05
* Bigint: new functions of_int and to_int, 2nd arg of pow in intGravatar letouzey2012-08-02
* Getting rid of the undocumented [complete] tactic, which wasGravatar ppedrot2012-07-19
* Fixes r15610 (A new status Unsafe in Interface).Gravatar aspiwack2012-07-13
* Ring_polynom : a restricted simpl instead of a unfold;foldGravatar letouzey2012-07-07
* Extraction: Hashtbl.replace uses less ressources than Hashtbl.add (fix #2824)Gravatar letouzey2012-07-05
* Legacy Ring and Legacy Field migrated to contribsGravatar letouzey2012-07-05
* rewrite_db : a first attempt at using rewrite_strat for a quicker autorewriteGravatar letouzey2012-07-05
* More cleanup in Ring_polynom and EnvRingGravatar letouzey2012-07-05
* Kills the useless tactic annotations "in |- *"Gravatar letouzey2012-07-05
* Open Local Scope ---> Local Open Scope, same with Notation and aliiGravatar letouzey2012-07-05
* ZArith + other : favor the use of modern names instead of compat notationsGravatar letouzey2012-07-05
* Cleaning opening of the standard List module.Gravatar ppedrot2012-06-28
* Replace nat indices with positive one in Btauto.Gravatar ppedrot2012-06-28
* Added an indirection with respect to Loc in Compat. As many [open Compat]Gravatar ppedrot2012-06-22
* Internalization of pattern is done in two phases.Gravatar pboutill2012-06-14
* Changed encoding from ISO-8859-1 to UTF-8 for some remaining gallina files.Gravatar ppedrot2012-06-12
* More cleaningGravatar ppedrot2012-06-01
* Cleaning Pp.ppnl useGravatar ppedrot2012-06-01
* Getting rid of Pp.msgnl and Pp.message.Gravatar ppedrot2012-06-01
* Getting rid of Pp.msgGravatar ppedrot2012-05-30
* More uniformisation in Pp.warn functions.Gravatar ppedrot2012-05-30
* remove many excessive open Util & Errors in mli'sGravatar letouzey2012-05-29
* place all files specific to camlp4 syntax extensions in grammar/Gravatar letouzey2012-05-29
* 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
* Stuff about notation_constr (ex-aconstr) now in notation_ops.mlGravatar letouzey2012-05-29
* slim down a bit genarg.ml (pr_intro_pattern forgotten there)Gravatar letouzey2012-05-29
* Pattern as a mli-only file, operations in PatternopsGravatar letouzey2012-05-29
* New files intf/constrexpr.mli and intf/notation_term.mli out of TopconstrGravatar letouzey2012-05-29
* Glob_term now mli-only, operations now in Glob_opsGravatar letouzey2012-05-29
* Tacexpr as a mli-only, the few functions there are now in TacopsGravatar 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
* Decl_kinds becomes a pure mli file, remaining ops in new file kindops.mlGravatar letouzey2012-05-29
* Vernacexpr is now a mli-only file, locality stuff now in locality.mlGravatar letouzey2012-05-29
* Fix ocamlbuild compilation: remove subtac from *.itargetGravatar letouzey2012-04-23
* correct abort in Function when a proof of inversion failsGravatar letouzey2012-04-23
* Corrects a (very) longstanding bug of tactics. As is were, tactic expectingGravatar aspiwack2012-04-18
* Remove the Dp plugin.Gravatar gmelquio2012-04-17
* "A -> B" is a notation for "forall _ : A, B".Gravatar pboutill2012-04-12
* lib directory is cut in 2 cma.Gravatar pboutill2012-04-12
* remove plugins/subtac/subtac.ml reintroduced by mistaked in a previous commitGravatar letouzey2012-04-12
* info_trivial, info_auto, info_eauto, and debug (trivial|auto)Gravatar letouzey2012-03-30
* Module names and constant/inductive names are now in two separate namespacesGravatar letouzey2012-03-26