index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
plugins
/
extraction
Age
Commit message (
Expand
)
Author
2020-04-20
Remove mod_constraints field of module body
Gaëtan Gilbert
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-15
[proof] Move proof_global functionality to Proof_global from Pfedit
Emilio Jesus Gallego Arias
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-03-18
Update headers in the whole code base.
Théo Zimmermann
2020-02-20
Fixing #11114 (anomaly with Extraction Implicit on records).
Hugo Herbelin
2020-02-18
Merge PR #11529: [build] Consolidate stdlib's .v files under a single directory.
Théo Zimmermann
2020-02-14
Use thunks to univ instead of lazy constr for template typing
Gaëtan Gilbert
2020-02-13
[build] Consolidate stdlib's .v files under a single directory.
Emilio Jesus Gallego Arias
2020-02-12
Remove Goptions.opt_name field
Gaëtan Gilbert
2020-01-30
Do not rely on Libobject for the current environment in extraction.
Pierre-Marie Pédrot
2020-01-30
Merge PR #11307: Remove the hacks relying on hardwired libobject tags.
Maxime Dénès
2020-01-08
Factorize ascii extraction in ExtrOcamlChar.v
Maxime Dénès
2020-01-08
Better extraction of string literals in Haskell
Maxime Dénès
2020-01-08
Reimplement string <-> char list conversions
Xavier Leroy
2020-01-08
Typo in comment
Xavier Leroy
2020-01-08
Rename ExtrOcamlStringPlus into ExtrOcamlNativeString
Xavier Leroy
2020-01-08
Avoid hardcoded paths in extraction
Maxime Dénès
2020-01-08
Avoid warning 40
Maxime Dénès
2020-01-08
Support extraction of Coq's string type to OCaml's string type, continued
Xavier Leroy
2020-01-08
Support extraction of Coq's string type to OCaml's string type
Xavier Leroy
2019-12-22
Remove the hacks relying on hardwired libobject tags.
Pierre-Marie Pédrot
2019-11-21
[coq] Untabify the whole ML codebase.
Emilio Jesus Gallego Arias
2019-11-01
Add some doc snippet in ExtrOCamlFloats.v
Erik Martin-Dorel
2019-11-01
Add extraction for primitive floats
Erik Martin-Dorel
2019-11-01
Add primitive float computation in Coq kernel
Guillaume Bertholon
2019-10-23
Merge PR #10897: Fix coq#4741: Extract Constant/Inductive with JSON
Vincent Laporte
2019-10-14
Fix coq#4741: Extract Constant/Inductive with JSON
Helge Bahmann
2019-10-14
Use kernel info from Global for Lib.sections_{depth,are_opened}
Gaëtan Gilbert
2019-09-04
Merge PR #10577: Fix #7348: extraction of dependent record projections
Maxime Dénès
2019-09-04
Merge PR #10612: Fix feedback levels
Emilio Jesus Gallego Arias
2019-08-29
Make sure that all query commands return a notice (not an info) feedback
Maxime Dénès
2019-08-10
[extraction] Fix #7191: Avoid unsound eta-reduction
Kazuhiko Sakaguchi
2019-07-31
Fix #7348: extraction of dependent record projections
Kazuhiko Sakaguchi
2019-07-22
[Int63] Implement all primitives in OCaml
Vincent Laporte
2019-07-22
[Extraction] Add support for primitive integers
Vincent Laporte
2019-07-11
Merge PR #10498: [api] Deprecate GlobRef constructors.
Gaëtan Gilbert
2019-07-08
[api] Deprecate GlobRef constructors.
Emilio Jesus Gallego Arias
2019-07-08
[core] [api] Support OCaml 4.08
Emilio Jesus Gallego Arias
2019-07-03
Merge PR #10442: Reify libobject containers
Emilio Jesus Gallego Arias
2019-06-28
Reify libobject containers
Maxime Dénès
2019-06-27
[extraction] Remove not very useful call to dumpglob.
Emilio Jesus Gallego Arias
2019-06-17
Merge PR #10362: Kernel-side delaying of polymorphic opaque constants
Gaëtan Gilbert
2019-06-17
Update ml-style headers to new year.
Théo Zimmermann
2019-06-17
Allow to delay polymorphic opaque constants.
Pierre-Marie Pédrot
2019-06-09
[proof] Move proofs that have an associated constant to `Lemmas`
Emilio Jesus Gallego Arias
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
[next]