index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
plugins
/
omega
Commit message (
Expand
)
Author
Age
*
Removing the old refine tactic from the Tactics module.
Pierre-Marie Pédrot
2016-05-17
*
Put the "generalize" tactic in the monad.
Pierre-Marie Pédrot
2016-05-16
*
Put the "clear" tactic into the monad.
Pierre-Marie Pédrot
2016-05-16
*
Removing dead code and unused opens.
Pierre-Marie Pédrot
2016-05-08
*
Removing the special status of generic entries defined by Coq itself.
Pierre-Marie Pédrot
2016-03-17
*
Getting rid of the "<:tactic< ... >>" quotations.
Pierre-Marie Pédrot
2016-02-24
*
merging conflicts with the original "trunk__CLEANUP__Context__2" branch
Matej Kosik
2016-02-15
|
\
*
|
Moving conversion functions to the new tactic API.
Pierre-Marie Pédrot
2016-02-15
|
*
CLEANUP: Context.{Rel,Named}.Declaration.t
Matej Kosik
2016-02-09
|
/
*
Merge branch 'v8.5'
Pierre-Marie Pédrot
2016-01-21
|
\
|
*
Update copyright headers.
Maxime Dénès
2016-01-20
*
|
Boxing the Goal.enter primitive into a record type.
Pierre-Marie Pédrot
2015-10-20
|
/
*
Fix some typos.
Guillaume Melquiond
2015-10-13
*
Safer typing primitives.
Pierre-Marie Pédrot
2015-05-13
*
Using tclZEROMSG instead of tclZERO in several places.
Pierre-Marie Pédrot
2015-04-23
*
Accomodating #4166 (providing "Require Import OmegaTactic" as a
Hugo Herbelin
2015-04-01
*
Update headers.
Maxime Dénès
2015-01-12
*
Switch the few remaining iso-latin-1 files to utf8
Pierre Letouzey
2014-12-09
*
Writing the raw introduction tactic in the new monad.
Pierre-Marie Pédrot
2014-11-05
*
A version of convert_concl and convert_hyp in new proof engine.
Hugo Herbelin
2014-10-09
*
Renaming goal-entering functions.
Pierre-Marie Pédrot
2014-09-06
*
Reorganization of tactics:
Hugo Herbelin
2014-08-18
*
Removing some tactic compatibility layer.
Pierre-Marie Pédrot
2014-08-01
*
Arith: full integration of the "Numbers" modular framework
Pierre Letouzey
2014-07-09
*
Now parsing rules of ML-declared tactics are only made available after the
Pierre-Marie Pédrot
2014-05-12
*
- Rename eq to equal in Univ, document new modules, set interfaces.
Matthieu Sozeau
2014-05-06
*
This commit adds full universe polymorphism and fast projections to Coq.
Matthieu Sozeau
2014-05-06
*
Removing useless try-with clauses in Goal.enter variants.
Pierre-Marie Pédrot
2014-04-25
*
Remove many superfluous 'open' indicated by ocamlc -w +33
Pierre Letouzey
2014-03-05
*
Proofview.Notations: Now that (>>=) is free, use it for tclBIND.
Arnaud Spiwack
2014-02-27
*
Less dependencies in Omega.
Pierre-Marie Pédrot
2014-02-08
*
Omega: avoiding distinct proof-terms on repeated identical runs
Pierre Letouzey
2014-01-10
*
Writing [cut] tactic using the new monad.
Pierre-Marie Pédrot
2013-12-02
*
Porting Tactics.assumption to the new engine.
ppedrot
2013-11-08
*
Made Proofview.Goal.hyps a named_context.
aspiwack
2013-11-02
*
Less use of the list-based interface for goal-bound tactics.
aspiwack
2013-11-02
*
Tachmach.New is now in Proofview.Goal.enter style.
aspiwack
2013-11-02
*
More Proofview.Goal.enter.
aspiwack
2013-11-02
*
Small syntax fix to be compatible with Ocaml 3.11.
aspiwack
2013-11-02
*
Removed spurious try/with in Proofview.Notation.(>>=) and (>>==).
aspiwack
2013-11-02
*
Clean-up: removed redundant notations (>>-) and (>>--) from Proofview.Notations.
aspiwack
2013-11-02
*
Getting rid of Goal.here, and all the related exceptions and combinators.
aspiwack
2013-11-02
*
Makes the new Proofview.tactic the basic type of Ltac.
aspiwack
2013-11-02
*
More monomorphic List.mem + List.assoc + ...
letouzey
2013-10-24
*
Turn many List.assoc into List.assoc_f
letouzey
2013-10-24
*
cList: a few alternative to hashtbl-based uniquize, distinct, subset
letouzey
2013-10-23
*
cList: set-as-list functions are now with an explicit comparison
letouzey
2013-10-23
*
Removing a bunch of generic equalities.
ppedrot
2013-09-27
*
Get rid of the uses of deprecated OCaml elements (still remaining compatible ...
xclerc
2013-09-19
*
Restrict (try...with...) to avoid catching critical exn (part 15)
letouzey
2013-03-13
[next]