index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
plugins
/
funind
/
recdef.ml
Age
Commit message (
Expand
)
Author
2021-01-04
Change the representation of kernel case.
Pierre-Marie Pédrot
2020-12-01
Fix a bug in funind.
Pierre-Marie Pédrot
2020-09-29
Applying ocamlformat.
Hugo Herbelin
2020-09-29
Almost fully moving funind to new proof engine.
Hugo Herbelin
2020-08-25
funind: stop using intro_using
Gaëtan Gilbert
2020-07-08
declare: Add [save_regular] API for obligation-ignoring proofs
Gaëtan Gilbert
2020-07-08
[obligations] Functionalize Program state
Emilio Jesus Gallego Arias
2020-07-06
Primitive persistent arrays
Maxime Dénès
2020-07-01
UIP in SProp
Gaëtan Gilbert
2020-06-26
[declare] Return list of declared global in Proof.save
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] [api] Removal of duplicated type aliases.
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-11
Merge PR #12273: Deprecate Refiner API
Emilio Jesus Gallego Arias
2020-05-07
[declare] Merge DeclareDef into Declare
Emilio Jesus Gallego Arias
2020-05-07
Remove call to Refiner API from Funind.
Pierre-Marie Pédrot
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-10
[ocamlformat] Enable for funind.
Emilio Jesus Gallego Arias
2020-03-18
Update headers in the whole code base.
Théo Zimmermann
2020-03-06
Fix #11738 : Funind using deprecated Coqlib API.
Pierre Courtieu
2020-02-07
Remove unsafe_type_of from funind
Gaëtan Gilbert
2020-02-07
various unsafe_type_of -> type_of_variable in funind
Gaëtan Gilbert
2019-11-01
Add primitive float computation in Coq kernel
Guillaume Bertholon
2019-10-25
[funind] Removed dead code.
Emilio Jesus Gallego Arias
2019-08-23
[lemmas] Cleanup users of default proof information.
Emilio Jesus Gallego Arias
2019-07-31
[funind] Port aux function to the new tactic engine.
Emilio Jesus Gallego Arias
2019-07-31
[funind] Move duplicated `observe_tac` function to indfun_common.
Emilio Jesus Gallego Arias
2019-07-11
Merge PR #10498: [api] Deprecate GlobRef constructors.
Gaëtan Gilbert
2019-07-09
[proof] Remove sign parameter to open_lemma.
Emilio Jesus Gallego Arias
2019-07-08
[api] Deprecate GlobRef constructors.
Emilio Jesus Gallego Arias
2019-07-07
[error] Remove special error printing pre-processing
Emilio Jesus Gallego Arias
2019-07-01
[decls] Remove goal_object_kind type.
Emilio Jesus Gallego Arias
2019-07-01
[declare] Separate kinds from entries in constant declaration
Emilio Jesus Gallego Arias
2019-07-01
[api] Refactor most of `Decl_kinds`
Emilio Jesus Gallego Arias
2019-06-28
Merge PR #10434: [declare] Fine tuning of Hook type.
Pierre-Marie Pédrot
2019-06-26
[stm] [vernac] Remove special ?proof parameter from vernac main path
Emilio Jesus Gallego Arias
2019-06-26
[declare] Fine tuning of Hook type.
Emilio Jesus Gallego Arias
2019-06-24
[api] Move `locality` from `library` to `vernac`.
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-24
Duplicate the type of constant entries in Proof_global.
Pierre-Marie Pédrot
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] Move declaration hooks to DeclareDef.
Emilio Jesus Gallego Arias
2019-06-12
[funind] Untabify; necessary to ease the review of subsequent work.
Emilio Jesus Gallego Arias
[next]