aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/evarutil.ml
Commit message (Expand)AuthorAge
* Fixing incorrect change to pattern-unification over Meta's introducedGravatar herbelin2011-11-06
* Continuing r14585 (ill-typed restriction bug).Gravatar herbelin2011-10-25
* Continuing r1492 (useless changes were inadvertantly committed)Gravatar herbelin2011-10-25
* New strategy to infer return predicate of match construct whenGravatar herbelin2011-10-25
* Fixing another bug revealing ill-typed use of evar restriction.Gravatar herbelin2011-10-24
* Fixing instance/filter mismatch in materialize_evar + documentation.Gravatar herbelin2011-10-24
* Partly reverting r14539 about fully expanding "let-in"s and not justGravatar herbelin2011-10-17
* More robust and uniform treatment of aliases in evarutil.mlGravatar herbelin2011-10-10
* Applied the trick of Chung-Kil Hur to solve second-order matchingGravatar herbelin2011-10-10
* Fixing buggy abberant code for Evarutil.expand_evarGravatar herbelin2011-10-10
* Passed conv_algo to evar_define and move call to solve_refl toGravatar herbelin2011-10-10
* Fix nf_evars_undefinedGravatar msozeau2011-08-03
* Evarutil: replace generic list_distinct on constr by constr_list_distinctGravatar puech2011-07-29
* Evarutil: replaced some generic = on constr by destructorsGravatar puech2011-07-29
* Evarutil: generic equality on constr replaced by destructorsGravatar puech2011-07-29
* Evarutil: generic equality on constr replaced by eq_constr (x2)Gravatar puech2011-07-29
* Evarutil: generic equality on constr replaced by eq_constrGravatar puech2011-07-29
* Added full pattern-unification on Meta for tactic unification.Gravatar herbelin2011-06-13
* Fixes in pruning, do not fail if pruning is impossible due to typing constrai...Gravatar msozeau2011-06-10
* More fixes in pruning/restriction of evars during unification.Gravatar msozeau2011-06-09
* Fixes in pruning in unification.Gravatar msozeau2011-06-08
* - Fix restrict_hyps to not allow filtering on a variable required to typechec...Gravatar msozeau2011-06-07
* - Make typeclass transparency information directly availableGravatar msozeau2011-04-13
* - Remove create_evar_defsGravatar msozeau2011-04-13
* Catch NotArity exception and transform it into an anomaly in retyping.Gravatar msozeau2011-04-11
* - Fix solve_simpl_eqn which was cheking instances types in the wrong environm...Gravatar msozeau2011-03-23
* Tentative to make unification check types at every instanciation of anGravatar msozeau2011-03-11
* - Better error messages taking unif. constraints into account.Gravatar msozeau2011-03-11
* Reverted commit r13893 about propagation of more informativeGravatar herbelin2011-03-07
* Added propagation of evars unification failure reasons for betterGravatar herbelin2011-03-07
* Added a table for using reserved names for binding names to typesGravatar herbelin2011-03-05
* Improved define_evar_as_lambda which was creating an unrelated new evarGravatar herbelin2011-03-05
* Instantiate evar by a lambda when "?n args" has to unify with ProdGravatar herbelin2011-03-05
* In evars_of_term and co, visit array c in Evar(_,c) (sequel to r13809)Gravatar letouzey2011-02-11
* Repair Class_tactics.split_evars, broken by r13717 (should fix #2481)Gravatar letouzey2011-02-03
* Rename rawterm.ml into glob_term.mlGravatar glondu2010-12-23
* Speed-up refine by avoiding some calls to Evd.foldGravatar letouzey2010-09-30
* Some dead code removal, thanks to Oug analyzerGravatar letouzey2010-09-24
* Updated all headers for 8.3 and trunkGravatar herbelin2010-07-24
* Fix (part of) bug #2347, de Bruijn bug in Program's pretyper.Gravatar msozeau2010-06-30
* Made tclABSTRACT normalize evars before saying it does not supportGravatar herbelin2010-06-29
* Added rudimentary support for using constructors from the explicitGravatar herbelin2010-06-12
* Fixed a bug in evarutil.ml (wrong env of a postponed conversion problem).Gravatar herbelin2010-06-12
* Mainly made that evarconv is able to solve "?n = (fun x => x) ?n" (sic).Gravatar herbelin2010-06-11
* Fixing Derive Inversion for new proof engineGravatar herbelin2010-05-26
* Improved the efficiency of evars traverals thanks to a split ofGravatar herbelin2010-05-13
* Remove the svn-specific $Id$ annotationsGravatar letouzey2010-04-29
* Here comes the commit, announced long ago, of the new tactic engine.Gravatar aspiwack2010-04-22
* Fixed bugs from commit 12954 on unification complexityGravatar herbelin2010-04-20
* Reduced the complexity of evar instantiations from O(n^3) to less than O(n^2).Gravatar herbelin2010-04-19