index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
plugins
/
ltac
Age
Commit message (
Expand
)
Author
2020-05-07
Deprecate the legacy tacticals from module Refiner.
Pierre-Marie Pédrot
2020-05-07
Port Evar_tactics to the new API.
Pierre-Marie Pédrot
2020-05-07
Export API to recover values out of Ltac application.
Pierre-Marie Pédrot
2020-05-07
Add helper API to define low-level Ltac functions.
Pierre-Marie Pédrot
2020-05-06
Moving lazymatch and multimatch to simple identifiers.
Hugo Herbelin
2020-05-06
Stop keeping outdated static list of keywords.
Hugo Herbelin
2020-05-06
Documenting plugin/tactic/stdlib keywords in corresponding chapters.
Hugo Herbelin
2020-05-02
Move tclWRAPFINALLY to profile_ltac
Jason Gross
2020-05-02
Decrease LtacProf overhead when not profiling
Jason Gross
2020-05-02
LtacProf now handles multi-success backtracking
Jason Gross
2020-04-28
Return an option in lookup_scheme.
Pierre-Marie Pédrot
2020-04-23
Merge PR #12130: [declare] [tactics] Move declare to `vernac`
Pierre-Marie Pédrot
2020-04-21
Merge PR #11896: Use lists instead of arrays in evar instances.
Maxime Dénès
2020-04-21
[declare] [tactics] Move declare to `vernac`
Emilio Jesus Gallego Arias
2020-04-21
[hints] Move and split Hint Declaration AST to vernac
Emilio Jesus Gallego Arias
2020-04-16
Merge PR #11861: [declare] [rewrite] Use high-level declare API
Pierre-Marie Pédrot
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-13
pass filters around
Gaëtan Gilbert
2020-04-11
[dune] [stdlib] Build the standard library natively with Dune.
Emilio Jesus Gallego Arias
2020-04-06
Clean and fix definitions of options.
Théo Zimmermann
2020-04-06
Use lists instead of arrays in evar instances.
Pierre-Marie Pédrot
2020-04-02
Merge PR #12002: Cleanup tactic_option a bit
Pierre-Marie Pédrot
2020-04-02
Cleanup tactic_option a bit
Gaëtan Gilbert
2020-03-31
Try only using TC for conversion in cominductive (not great but let's see)
Gaëtan Gilbert
2020-03-31
[declare] [rewrite] Use high-level declare API, part II.
Emilio Jesus Gallego Arias
2020-03-31
[declare] [rewrite] Use high-level declare API, part I.
Emilio Jesus Gallego Arias
2020-03-31
Merge PR #11647: [rfc] Consolidation of parsing interfaces
Pierre-Marie Pédrot
2020-03-26
Removing deprecated destruct syntax _eqn.
Hugo Herbelin
2020-03-25
[pcoq] Inline the exported Gramlib interface instead of exposing it as G
Emilio Jesus Gallego Arias
2020-03-25
[parsing] Remove redundant interfaces from Pcoq
Emilio Jesus Gallego Arias
2020-03-25
[parsing] Remove extend AST in favor of gramlib constructors
Emilio Jesus Gallego Arias
2020-03-25
[parsing] Make grammar rules private.
Emilio Jesus Gallego Arias
2020-03-25
[parsing] Make grammar extension type private.
Emilio Jesus Gallego Arias
2020-03-22
Centralizing all kinds of numeral string management in numTok.ml.
Hugo Herbelin
2020-03-19
Merge PR #11735: Deprecating catchable_exception
Pierre-Marie Pédrot
2020-03-18
Merge PR #11559: Remove year in headers.
Hugo Herbelin
2020-03-18
Update headers in the whole code base.
Théo Zimmermann
2020-03-18
Use a 3-valued flag for hint locality.
Pierre-Marie Pédrot
2020-03-18
Hack a non-superglobal mode for hints.
Pierre-Marie Pédrot
2020-03-13
Removing catchable_exception test in tclOR/tclORELSE.
Hugo Herbelin
2020-03-13
Replacing catchable_exception by noncritical in try-with blocks.
Hugo Herbelin
2020-03-08
Merge PR #11578: [exn] Keep information from multiple extra exn handlers
Pierre-Marie Pédrot
2020-03-05
Merge PR #11522: Adding an alias `pose proof (x:=t)` for `pose proof t as x` ...
Pierre-Marie Pédrot
2020-03-04
Merge PR #11380: [exninfo] Deprecate aliases for exception re-raising.
Pierre-Marie Pédrot
2020-03-04
Merge PR #11709: Deprecate the "prolog" tactic.
Théo Zimmermann
2020-03-03
[exn] Keep information from multiple extra exn handlers
Emilio Jesus Gallego Arias
2020-03-03
[exninfo] Deprecate aliases for exception re-raising.
Emilio Jesus Gallego Arias
2020-03-03
Adding an alias "pose proof (x:=a)" for "pose proof a as x".
Hugo Herbelin
[prev]
[next]