aboutsummaryrefslogtreecommitdiff
path: root/plugins
AgeCommit message (Expand)Author
2012-05-29New files intf/constrexpr.mli and intf/notation_term.mli out of Topconstrletouzey
2012-05-29Glob_term now mli-only, operations now in Glob_opsletouzey
2012-05-29Tacexpr as a mli-only, the few functions there are now in Tacopsletouzey
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-05-29Decl_kinds becomes a pure mli file, remaining ops in new file kindops.mlletouzey
2012-05-29Vernacexpr is now a mli-only file, locality stuff now in locality.mlletouzey
2012-04-23Fix ocamlbuild compilation: remove subtac from *.itargetletouzey
2012-04-23correct abort in Function when a proof of inversion failsletouzey
2012-04-18Corrects a (very) longstanding bug of tactics. As is were, tactic expectingaspiwack
2012-04-17Remove the Dp plugin.gmelquio
2012-04-12"A -> B" is a notation for "forall _ : A, B".pboutill
2012-04-12lib directory is cut in 2 cma.pboutill
2012-04-12remove plugins/subtac/subtac.ml reintroduced by mistaked in a previous commitletouzey
2012-03-30info_trivial, info_auto, info_eauto, and debug (trivial|auto)letouzey
2012-03-26Module names and constant/inductive names are now in two separate namespacesletouzey
2012-03-23A unified backtrack mechanism, with a basic "Show Script" as side-effectletouzey
2012-03-20Fixing alpha-conversion bug #2723 introduced in r12485-12486.herbelin
2012-03-18Fixing bug #2732 (anomaly when using the tolerance for writingherbelin
2012-03-14Fix merge.msozeau
2012-03-14Revise API of understand_ltac to be parameterized by a flag for resolution of...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-14Everything compiles again.msozeau
2012-03-14Second step of integration of Program:msozeau
2012-03-14Remove support for "abstract typing constraints" that requires unicity of sol...msozeau
2012-03-02Glob_term.predicate_pattern: No number of parameters with letins.pboutill
2012-03-02Noise for nothingpboutill
2012-03-01New version of recdef :jforest
2012-03-01various corrections in invfun due to a modification in inductionjforest
2012-02-29correcting a little bug in invfun.mljforest
2012-02-29correction of bug 2457jforest
2012-02-29In the syntax of pattern matching, "in" clauses are patterns.pboutill
2012-02-20Correct application of head reduction.msozeau
2012-02-15Avoid retrying uncessarily to prove independent remaining obligations in Prog...msozeau
2012-02-15Avoid unnecessary normalizations w.r.t. evars in Program.msozeau
2012-02-14- Fix dependency computation in eterm to not consider filtered variables.msozeau
2012-02-03correcting inversion in list of generated tcc of Functionletouzey
2012-01-31Fix camlp4 compilationpboutill
2012-01-30Added an pattern / occurence syntax for vm_compute.ppedrot
2012-01-23Fix for Program Instance not separately checking the resolution of evars of t...msozeau
2012-01-23Another quick hack that works this time, to handle printing of locality in Pr...ppedrot
2012-01-20Reverted previous commit, which broke library compilation.ppedrot
2012-01-20This is a quick hack to permit the parsing of the locality flag in the Progra...ppedrot
2012-01-17Fixed the pretty-printing of the Program plugin.ppedrot
2012-01-14coq_micromega.ml: fix order of recursive calls to rconstantglondu
2012-01-14More newlines in debugging output of psatzlglondu
2012-01-13Added a Btauto plugin, that solves boolean tautologies.ppedrot
2012-01-12Fix typoglondu
2011-12-16Moving bullets (-, +, *) into stand-alone commands instead of beingcourtieu