aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.ml
Commit message (Expand)AuthorAge
* Fix bug #4780: universe leak in letin_tacGravatar Matthieu Sozeau2016-07-20
* errors.ml renamed into cErrors.ml (avoid clash with an OCaml compiler-lib mod...Gravatar Pierre Letouzey2016-07-03
* Add and document match, fix and cofix reduction flags.Gravatar Maxime Dénès2016-07-01
* Separate flags for fix/cofix/match reduction and clean reduction function names.Gravatar Maxime Dénès2016-07-01
* A new infrastructure for warnings.Gravatar Maxime Dénès2016-06-29
* Shrink Proofs/Obligations by default and deprecateGravatar Matthieu Sozeau2016-06-27
* Optimization in the subst tactic.Gravatar Pierre-Marie Pédrot2016-06-24
* Optimization in the subst tactic.Gravatar Pierre-Marie Pédrot2016-06-24
* Small optimization in clear_body.Gravatar Pierre-Marie Pédrot2016-06-20
* Adding an "as" clause to specialize.Gravatar Hugo Herbelin2016-06-18
* Exporting a generic argument induction_arg. As a consequence,Gravatar Hugo Herbelin2016-06-18
* A cleaning phase around delayed induction arg + exporting force_induction_arg.Gravatar Hugo Herbelin2016-06-18
* Adding eintros to respect the e- prefix policy.Gravatar Hugo Herbelin2016-06-18
* A stronger invariant on the syntax of TacAssert, what allows for aGravatar Hugo Herbelin2016-06-16
* Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-06-13
|\
| * Fixing a try with in apply that has become too weak in 8.5.Gravatar Hugo Herbelin2016-06-11
* | Fixing #4787 (Unset Bracketing Last Introduction Pattern not working).Gravatar Hugo Herbelin2016-06-07
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-06-01
|\|
* | Feedback cleanupGravatar Emilio Jesus Gallego Arias2016-05-31
| * Fix bug #4746: Anomaly: Evar ?X10 was not declared.Gravatar Pierre-Marie Pédrot2016-05-29
* | Removing some compatibility layers in Tactics.Gravatar Pierre-Marie Pédrot2016-05-17
* | Put the "move" tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-17
* | Put the "change" tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "specialize_eq" tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "generalize dependent" tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "generalize" tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "cofix" tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "*_cast_no_check" tactics in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "exact" family of tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "fix" tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "exact_constr" tactic in the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Put the "clear" tactic into the monad.Gravatar Pierre-Marie Pédrot2016-05-16
* | Removing dead code and unused opens.Gravatar Pierre-Marie Pédrot2016-05-08
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-05-04
|\|
| * Fix bug #4707: clearbody much slower in 8.5pl1.Gravatar Pierre-Marie Pédrot2016-05-03
* | Revert "In the short term, stronger invariant on the syntax of TacAssert, what"Gravatar Hugo Herbelin2016-04-27
* | In the short term, stronger invariant on the syntax of TacAssert, whatGravatar Hugo Herbelin2016-04-27
* | Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2016-04-09
|\|
| * Fixing the "No applicable tactic" non informative error messageGravatar Hugo Herbelin2016-04-03
* | Moving Refine to its proper module.Gravatar Pierre-Marie Pédrot2016-03-20
* | Making Proofview independent of Logic.Gravatar Pierre-Marie Pédrot2016-03-20
* | merging conflicts with the original "trunk__CLEANUP__Context__2" branchGravatar Matej Kosik2016-02-15
|\ \
* | | Using monotonic types for conversion functions.Gravatar Pierre-Marie Pédrot2016-02-15
* | | Code factorization of tactic "unfold_body".Gravatar Pierre-Marie Pédrot2016-02-15
* | | More conversion functions in the new tactic API.Gravatar Pierre-Marie Pédrot2016-02-15
* | | Moving conversion functions to the new tactic API.Gravatar Pierre-Marie Pédrot2016-02-15
* | | Renaming functions in Typing to stick to the standard e_* scheme.Gravatar Pierre-Marie Pédrot2016-02-15
* | | Monotonizing the Evarutil module.Gravatar Pierre-Marie Pédrot2016-02-15
| * | CLEANUP: Context.{Rel,Named}.Declaration.tGravatar Matej Kosik2016-02-09
|/ /
* | Fixing a use of "clear" on an non-existing hypothesis in intro-patterns.Gravatar Hugo Herbelin2016-01-22