index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
pretyping
/
cases.ml
Commit message (
Expand
)
Author
Age
*
Added an indirection with respect to Loc in Compat. As many [open Compat]
ppedrot
2012-06-22
*
Glob_term now mli-only, operations now in Glob_ops
letouzey
2012-05-29
*
Evar_kinds.mli containing former Evd.hole_kind, avoid deps on Evd
letouzey
2012-05-29
*
Impossible branches inference fixup (bug 2761)
pboutill
2012-05-11
*
Fix bugs related to Program integration.
msozeau
2012-03-19
*
Revise API of understand_ltac to be parameterized by a flag for resolution of...
msozeau
2012-03-14
*
Merge fixes
msozeau
2012-03-14
*
Everything compiles again.
msozeau
2012-03-14
*
Second step of integration of Program:
msozeau
2012-03-14
*
Remove support for "abstract typing constraints" that requires unicity of sol...
msozeau
2012-03-14
*
A bit of cleaning: unifying push_rels and push_rel_context.
herbelin
2012-03-13
*
Glob_term.predicate_pattern: No number of parameters with letins.
pboutill
2012-03-02
*
Noise for nothing
pboutill
2012-03-02
*
Inductiveops.nb_*{,_env} cleaning
pboutill
2012-01-16
*
Introducing a notion of evar candidates to be used when an evar is
herbelin
2011-12-16
*
Fixed a small regression in pattern-matching compilation introduced in
herbelin
2011-12-04
*
Finally used typing to decide whether an alias needs to be expanded or
herbelin
2011-11-28
*
Fixing dependencies postprocessing bug in pattern-matching compilation.
herbelin
2011-11-28
*
Fixed a bug in postprocessing dependencies in pattern-matching compilation
herbelin
2011-11-26
*
Extend the computation of dependencies in pattern-matching compilation
herbelin
2011-11-21
*
Add matching on non-inductive types in building an inversion problem
herbelin
2011-11-21
*
Old naming bug in pattern-matching compilation: names in the
herbelin
2011-11-21
*
Inlining let-in (i.e. trace of aliases) in extract_predicate for what
herbelin
2011-11-21
*
In pattern-matching compilation, now taking into account the dependencies
herbelin
2011-11-21
*
Optimizing the compilation of unused aliases in pattern-matching.
herbelin
2011-11-21
*
Simplifying history management in pattern-matching compilation.
herbelin
2011-11-21
*
Fixing postprocessing bugs in pattern-matching compilation.
herbelin
2011-11-21
*
Removing stuff about alias dependencies now become useless.
herbelin
2011-11-21
*
Changed the way to detect if an "as" patterns is expanded or not. The
herbelin
2011-11-21
*
Dead code + refreshing some comments in cases.ml.
herbelin
2011-11-21
*
Fixing new bug introduced in r14665 when fixing bug #1834.
herbelin
2011-11-17
*
Adding postprocessing to remove "commutative cuts" expansions in
herbelin
2011-11-16
*
Changed the way find_dependencies_signature is working so that it
herbelin
2011-11-16
*
De Bruijn indices bug in pattern matching compilation in the presence
herbelin
2011-11-16
*
Old generalization bug in pattern-matching: names were considered the
herbelin
2011-11-16
*
Fixing bug #1834 (de Bruijn indices bug in pattern-matching compilation).
herbelin
2011-11-16
*
Old typing bug in pattern-matching compilation (apparently w/o
herbelin
2011-11-16
*
Specialization of tomatch in pattern-matching compilation was done too
herbelin
2011-11-16
*
A bit of documentation around cases.ml + ML modules uselessly open
herbelin
2011-11-16
*
Fixing dependencies lifting bug in pattern-matching compilation
herbelin
2011-11-16
*
Fixing use of type constraint for refining the "return" clause of "match".
herbelin
2011-10-25
*
New strategy to infer return predicate of match construct when
herbelin
2011-10-25
*
It happens that the type inference algorithm (pretyping) did not check
herbelin
2011-10-05
*
Two bugs in pattern-matching compilation:
herbelin
2011-08-08
*
Cases: generic equality on constr replaced by destructors
puech
2011-07-29
*
Fix inductive_template building ill-typed evars, and update test-suite scripts
msozeau
2011-03-13
*
Tentative to make unification check types at every instanciation of an
msozeau
2011-03-11
*
More {raw => glob} changes for consistency
glondu
2010-12-24
*
Rename rawterm.ml into glob_term.ml
glondu
2010-12-23
*
Change of nomenclature: rawconstr -> glob_constr
glondu
2010-12-23
[next]