index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
plugins
/
derive
Age
Commit message (
Expand
)
Author
2021-03-03
[build] Split stdlib to it's own opam package.
Emilio Jesus Gallego Arias
2020-06-26
[declare] Remove Proof_ending from the public API
Emilio Jesus Gallego Arias
2020-06-26
[declare] Improve organization of proof/constant information.
Emilio Jesus Gallego Arias
2020-06-26
[declare] Reify Proof.t API into the Proof module.
Emilio Jesus Gallego Arias
2020-06-26
[declare] Move udecl to Info structure.
Emilio Jesus Gallego Arias
2020-06-26
[declare] Remove Lemmas module
Emilio Jesus Gallego Arias
2020-06-26
[declare] Move proof information to declare.
Emilio Jesus Gallego Arias
2020-05-18
[declare] Grand unification of the proof save path.
Emilio Jesus Gallego Arias
2020-04-15
[declare] Rename `Declare.t` to `Declare.Proof.t`
Emilio Jesus Gallego Arias
2020-04-15
[proof] Merge `Proof_global` into `Declare`
Emilio Jesus Gallego Arias
2020-04-11
[dune] [stdlib] Build the standard library natively with Dune.
Emilio Jesus Gallego Arias
2020-03-18
Update headers in the whole code base.
Théo Zimmermann
2020-02-13
[build] Consolidate stdlib's .v files under a single directory.
Emilio Jesus Gallego Arias
2019-07-01
[decls] Remove goal_object_kind type.
Emilio Jesus Gallego Arias
2019-07-01
[api] Refactor most of `Decl_kinds`
Emilio Jesus Gallego Arias
2019-06-24
[lemmas] [proof] Split proof kinds into per-layer components.
Emilio Jesus Gallego Arias
2019-06-24
[proof] Remove duplicated universe polymorphic from decl_kinds
Emilio Jesus Gallego Arias
2019-06-24
[lemmas] Turn Lemmas.info into a proper type with constructor.
Emilio Jesus Gallego Arias
2019-06-20
Merge PR #9645: [proof] Remove terminator type, unifying regular and obligati...
Pierre-Marie Pédrot
2019-06-17
Update ml-style headers to new year.
Théo Zimmermann
2019-06-17
[proof] Remove terminator type, unifying regular and obligation ones.
Emilio Jesus Gallego Arias
2019-06-17
[proof] drop parameter from terminator type
Emilio Jesus Gallego Arias
2019-06-17
[proofs] Store hooks in the proof object.
Emilio Jesus Gallego Arias
2019-06-13
Merge PR #10319: [STM] Only VtSideeff can be VtNow/VtLater
Enrico Tassi
2019-06-11
Remove the side-effect role from the kernel.
Pierre-Marie Pédrot
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-09
[save_proof] Make terminator API internal.
Emilio Jesus Gallego Arias
2019-06-09
[proof] Move proofs that have an associated constant to `Lemmas`
Emilio Jesus Gallego Arias
2019-06-08
Cleaning the status of Local Definition and similar.
Hugo Herbelin
2019-06-04
Rename Proof_global.{pstate -> t}
Gaëtan Gilbert
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-06-04
Proof_global: pass only 1 pstate when we don't want the proof stack
Gaëtan Gilbert
2019-05-14
Allow run_tactic to return a value, remove hack from ltac2
Gaëtan Gilbert
2019-03-27
[plugins] [derive] Adapt to removal of imperative proof state.
Emilio Jesus Gallego Arias
2019-03-14
Add relevance marks on binders.
Gaëtan Gilbert
2019-02-05
Make Program a regular attribute
Maxime Dénès
2019-01-24
[STM] explicit handling of parsing states
Enrico Tassi
2018-12-09
[doc] Enable Warning 50 [incorrect doc comment] and fix comments.
Emilio Jesus Gallego Arias
2018-11-17
[vernacextend] Consolidate extension points API
Emilio Jesus Gallego Arias
2018-10-02
Make the coqpp VERNAC EXTEND behave as the non-FUNCTIONAL camlp5 one.
Pierre-Marie Pédrot
2018-10-02
Port g_derive to coqpp.
Pierre-Marie Pédrot
2018-09-05
[build] Preliminary support for building Coq with `dune`.
Emilio Jesus Gallego Arias
2018-05-23
[api] Move `opacity_flag` to `Proof_global`.
Emilio Jesus Gallego Arias
2018-02-27
Update headers following #6543.
Théo Zimmermann
2018-02-17
Change references to CAMLP4 to CAMLP5 to be more accurate since we no
Jim Fehrle
2017-12-15
[econstr] Switch constrintern API to non-imperative style.
Emilio Jesus Gallego Arias
2017-11-06
[api] Move structures deprecated in the API to the core.
Emilio Jesus Gallego Arias
2017-10-17
[stm] Remove state-handling from Futures.
Emilio Jesus Gallego Arias
[next]