index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
plugins
/
ltac
/
g_ltac.mlg
Age
Commit message (
Expand
)
Author
2021-01-07
Use nat_or_var for fail/gfail
Jim Fehrle
2020-11-20
Use nat_or_var where negative values don't make sense
Jim Fehrle
2020-11-12
Revert to "using" not being a keyword in -noinit mode.
Théo Zimmermann
2020-11-12
Add support for Proof using in -noinit mode.
Théo Zimmermann
2020-10-29
Use same code for "Print Ltac foo" and "Print foo" when "foo" is an Ltac.
Hugo Herbelin
2020-10-27
Rename misc nonterminals
Jim Fehrle
2020-10-27
Rename tactic_expr -> ltac_expr
Jim Fehrle
2020-10-27
Rename operconstr -> term
Jim Fehrle
2020-10-26
Improve tactic interpreter registration API a bit
Gaëtan Gilbert
2020-10-09
Merge PR #13088: [stm] move par: to comTactic
coqbot-app[bot]
2020-10-09
[stm] move par: implementation to vernac/comTactic and stm/partac
Enrico Tassi
2020-10-04
Remove prefixes on nonterminal names, e.g. "constr:" and "Prim."
Jim Fehrle
2020-09-22
Fixes #9716, #13004: don't drop the qualifier of quotations at printing time.
Hugo Herbelin
2020-09-11
Turn integer into natural in several mlgs
Pierre Roux
2020-06-26
[declare] Move proof information to declare.
Emilio Jesus Gallego Arias
2020-05-30
Remove info tactic, deprecated in 8.5
Jim Fehrle
2020-05-13
Merge PR #12229: Hopefully consensual cleaning of keywords
Théo Zimmermann
2020-05-07
[declare] Merge DeclareDef into Declare
Emilio Jesus Gallego Arias
2020-05-06
Moving lazymatch and multimatch to simple identifiers.
Hugo Herbelin
2020-04-21
[hints] Move and split Hint Declaration AST to vernac
Emilio Jesus Gallego Arias
2020-04-15
[declare] Rename `Declare.t` to `Declare.Proof.t`
Emilio Jesus Gallego Arias
2020-04-15
[proof] Merge `Pfedit` into proofs.
Emilio Jesus Gallego Arias
2020-04-15
[proof] Merge `Proof_global` into `Declare`
Emilio Jesus Gallego Arias
2020-04-06
Clean and fix definitions of options.
Théo Zimmermann
2020-03-18
Update headers in the whole code base.
Théo Zimmermann
2020-03-01
Refactor lookaheads using DSL
Maxime Dénès
2020-02-12
Remove Goptions.opt_name field
Gaëtan Gilbert
2019-11-21
[coq] Untabify the whole ML codebase.
Emilio Jesus Gallego Arias
2019-07-29
Tentatively providing a localization function to ad-hoc camlp5 parsers.
Pierre-Marie Pédrot
2019-06-19
Merge PR #10239: Deprecate grammar entry "intropattern" in tactic notations i...
Théo Zimmermann
2019-06-17
Update ml-style headers to new year.
Théo Zimmermann
2019-06-16
Deprecate "intro_pattern" in tactic notations in favor of "simple_intropattern".
Hugo Herbelin
2019-06-11
STM: encode in static types that vernac_when is only used when VtSideff
Gaëtan Gilbert
2019-06-09
[proof] Uniformize Proof_global API
Emilio Jesus Gallego Arias
2019-06-04
Alternate syntax for ![]: VERNAC EXTEND Foo STATE proof
Gaëtan Gilbert
2019-06-04
coqpp: add new ![] specifiers for structured proof interaction
Gaëtan Gilbert
2019-03-27
[coqpp] [ltac] Adapt to removal of imperative proof state.
Emilio Jesus Gallego Arias
2019-03-20
Stop accessing proof env via Pfedit in printers
Maxime Dénès
2019-01-24
[STM] explicit handling of parsing states
Enrico Tassi
2018-11-27
Merge PR #9046: Goptions.declare_* functions return unit instead of a write_f...
Emilio Jesus Gallego Arias
2018-11-23
Remove the unsafe camlp5 API from the Coq codebase.
Pierre-Marie Pédrot
2018-11-23
s/let _ =/let () =/ in some places (mostly goptions related)
Gaëtan Gilbert
2018-11-19
Merge PR #9003: [vernacextend] Consolidate extension points API
Pierre-Marie Pédrot
2018-11-17
[vernacextend] Consolidate extension points API
Emilio Jesus Gallego Arias
2018-11-17
[ltac] Use CAst nodes in the tactic AST.
Emilio Jesus Gallego Arias
2018-11-02
coqpp VERNAC EXTEND uses #[ att = attribute; ] syntax
Gaëtan Gilbert
2018-11-02
Command driven attributes.
Gaëtan Gilbert
2018-11-02
Move attributes out of vernacinterp to new attributes module
Gaëtan Gilbert
2018-10-15
Port remaining EXTEND ml4 files to coqpp.
Pierre-Marie Pédrot