aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins
Commit message (Expand)AuthorAge
* 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
* A unified backtrack mechanism, with a basic "Show Script" as side-effectGravatar letouzey2012-03-23
* Fixing alpha-conversion bug #2723 introduced in r12485-12486.Gravatar herbelin2012-03-20
* Fixing bug #2732 (anomaly when using the tolerance for writingGravatar herbelin2012-03-18
* Fix merge.Gravatar msozeau2012-03-14
* Revise API of understand_ltac to be parameterized by a flag for resolution of...Gravatar msozeau2012-03-14
* 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
* Everything compiles again.Gravatar msozeau2012-03-14
* Second step of integration of Program:Gravatar msozeau2012-03-14
* Remove support for "abstract typing constraints" that requires unicity of sol...Gravatar msozeau2012-03-14
* Glob_term.predicate_pattern: No number of parameters with letins.Gravatar pboutill2012-03-02
* Noise for nothingGravatar pboutill2012-03-02
* New version of recdef :Gravatar jforest2012-03-01
* various corrections in invfun due to a modification in inductionGravatar jforest2012-03-01
* correcting a little bug in invfun.mlGravatar jforest2012-02-29
* correction of bug 2457Gravatar jforest2012-02-29
* In the syntax of pattern matching, "in" clauses are patterns.Gravatar pboutill2012-02-29
* Correct application of head reduction.Gravatar msozeau2012-02-20
* Avoid retrying uncessarily to prove independent remaining obligations in Prog...Gravatar msozeau2012-02-15
* Avoid unnecessary normalizations w.r.t. evars in Program.Gravatar msozeau2012-02-15
* - Fix dependency computation in eterm to not consider filtered variables.Gravatar msozeau2012-02-14
* correcting inversion in list of generated tcc of FunctionGravatar letouzey2012-02-03
* Fix camlp4 compilationGravatar pboutill2012-01-31
* Added an pattern / occurence syntax for vm_compute.Gravatar ppedrot2012-01-30
* Fix for Program Instance not separately checking the resolution of evars of t...Gravatar msozeau2012-01-23
* Another quick hack that works this time, to handle printing of locality in Pr...Gravatar ppedrot2012-01-23
* Reverted previous commit, which broke library compilation.Gravatar ppedrot2012-01-20
* This is a quick hack to permit the parsing of the locality flag in the Progra...Gravatar ppedrot2012-01-20
* Fixed the pretty-printing of the Program plugin.Gravatar ppedrot2012-01-17