index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
plugins
/
funind
/
gen_principle.ml
Age
Commit message (
Expand
)
Author
2021-04-23
Merge PR #13965: [abbreviation] user syntax to set interp scope of argument
Pierre-Marie Pédrot
2021-04-19
Check for existence before using `Global.lookup_constant` instead of catching...
Lasse Blaauwbroek
2021-04-07
cleanup: less exceptions, removal of try_interp_name_alias
Enrico Tassi
2021-01-04
Change the representation of kernel case.
Pierre-Marie Pédrot
2020-12-21
Move evaluable_global_reference from Names to Tacred.
Pierre-Marie Pédrot
2020-10-21
Deprecate the non-qualified equality functions on kerpairs.
Pierre-Marie Pédrot
2020-10-08
Dropping the misleading int argument of Pp.h.
Hugo Herbelin
2020-09-29
Applying ocamlformat.
Hugo Herbelin
2020-09-29
Almost fully moving funind to new proof engine.
Hugo Herbelin
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-03
Merge PR #10390: UIP in SProp
Maxime Dénès
2020-07-01
[state] Consolidate state handling in Vernacstate
Emilio Jesus Gallego Arias
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-09
Merge PR #12241: [declare] Merge DeclareDef into Declare
Gaëtan Gilbert
2020-05-08
Merge PR #12121: Fixes #11903 and warns about non truly-recursive (co)fixpoints
Pierre-Marie Pédrot
2020-05-07
[declare] Merge DeclareDef into Declare
Emilio Jesus Gallego Arias
2020-05-03
[declare] Add deprecation notices for compat modules.
Emilio Jesus Gallego Arias
2020-05-03
[funind] Remove use of low-level entries in scheme generation.
Emilio Jesus Gallego Arias
2020-05-03
[funind] Make `build_functional_principle` use a functional evar_map
Emilio Jesus Gallego Arias
2020-05-01
Warn when a (co)fixpoint is not truly recursive.
Hugo Herbelin
2020-04-19
Merge PR #12033: Let coqdoc be informed by coq about binding variables (incid...
Lysxia
2020-04-15
Coqdoc: Exporting location and unique id for binding variables.
Hugo Herbelin
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-31
Merge PR #11915: [proof] Split delayed and regular proof closing functions
Pierre-Marie Pédrot
2020-03-31
Merge PR #11823: [funind] [cleanup] Remove unused function parameters
Pierre-Marie Pédrot
2020-03-31
[proof] Split delayed and regular proof closing functions, part II
Emilio Jesus Gallego Arias
2020-03-30
[declare] Fuse prepare and declare for the non-interactive path.
Emilio Jesus Gallego Arias
2020-03-30
[declareDef] More consistent handling of universe binders
Emilio Jesus Gallego Arias
2020-03-30
[declare] Make the type of closed entries opaque.
Emilio Jesus Gallego Arias
2020-03-30
[ComDefinition] Split program from regular declarations
Emilio Jesus Gallego Arias
2020-03-30
[proof] Miscellaneous cleanup on proof info handling
Emilio Jesus Gallego Arias
2020-03-19
[declare] Bring more consistency to parameters using labels
Emilio Jesus Gallego Arias
2020-03-18
Update headers in the whole code base.
Théo Zimmermann
2020-03-13
[funind] [cleanup] Remove unused function parameters
Emilio Jesus Gallego Arias
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-12-06
Moving the diversity of constr printers to a label style.
Hugo Herbelin
2019-11-01
Add primitive float computation in Coq kernel
Guillaume Bertholon
2019-10-25
[funind] Remove duplicate save function.
Emilio Jesus Gallego Arias
2019-09-29
Merge PR #10673: [lemmas] Cleanup users of default proof information.
Pierre-Marie Pédrot
[next]