aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/funind
Commit message (Expand)AuthorAge
* Glob_term now mli-only, operations now in Glob_opsGravatar 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
* correct abort in Function when a proof of inversion failsGravatar letouzey2012-04-23
* "A -> B" is a notation for "forall _ : A, B".Gravatar pboutill2012-04-12
* info_trivial, info_auto, info_eauto, and debug (trivial|auto)Gravatar letouzey2012-03-30
* 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
* Final part of moving Program code inside the main code. Adapted add_definitio...Gravatar msozeau2012-03-14
* Second step of integration of Program:Gravatar msozeau2012-03-14
* 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
* correcting inversion in list of generated tcc of FunctionGravatar letouzey2012-02-03
* Proof using ...Gravatar gareuselesinge2011-12-12
* Added a DEPRECATED flag in declaration of options. For now only two options a...Gravatar ppedrot2011-11-24
* Add type annotations around all calls to Libobject.declare_objectGravatar letouzey2011-11-02
* Remove dynamic stuff from constr_expr and glob_constrGravatar glondu2011-10-28
* Remove avoidable use of GDynamicGravatar glondu2011-10-27
* Fixing Equality.injectable which did not detect an equality withoutGravatar herbelin2011-10-22
* Fixing Implicit Tactic mode damaged by commit r14496 (see also bug #2612).Gravatar herbelin2011-10-05
* Added support for referring to subterms of the goal by pattern.Gravatar herbelin2011-09-26
* correction du bug 2047Gravatar jforest2011-09-09
* Recdef: replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* Functional_principles_types: replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* Relaxed the constraint introduced in r14190 that froze the existingGravatar herbelin2011-06-18
* Call process_vernac_interp_error before calling Errors.print inGravatar herbelin2011-06-10
* A new mechanism to handle errors.Gravatar aspiwack2011-05-13
* Revert "Add [Polymorphic] flag for defs"Gravatar msozeau2011-04-13
* Add [Polymorphic] flag for defsGravatar msozeau2011-04-13
* Lazy loading of opaque proofs: fast as -dont-load-proofs without its drawbacksGravatar letouzey2011-04-03
* Data structure telling implicits of local variables is a map in theGravatar pboutill2011-02-10
* Remove the "Boxed" syntaxes and the const_entry_boxed fieldGravatar letouzey2011-01-28
* ARGUMENT EXTEND: forbid TYPED simultaneously with {RAW,GLOB}_TYPEDGravatar glondu2010-12-25
* Rename mkR* smart constructors (mostly in funind)Gravatar glondu2010-12-25
* More {raw => glob} changes for consistencyGravatar glondu2010-12-24
* Rename files in funind to respect new conventionsGravatar glondu2010-12-24
* Rename rawterm.ml into glob_term.mlGravatar glondu2010-12-23
* Change of nomenclature: rawconstr -> glob_constrGravatar glondu2010-12-23
* Prepare change of nomenclature rawconstr -> glob_constrGravatar glondu2010-12-23
* An experimental support for open constrs in hints and in "using"Gravatar herbelin2010-10-31
* Auto-inlining of f_terminate in FunctionGravatar jforest2010-10-05
* Simplify tactic(_)-bound arguments in TACTIC EXTEND rulesGravatar glondu2010-09-30
* Remove some occurrences of "open Termops"Gravatar glondu2010-09-28
* Remove "init" label from Termops.it_mk* specialized functionsGravatar glondu2010-09-28