aboutsummaryrefslogtreecommitdiffhomepage
path: root/library/library.ml
Commit message (Expand)AuthorAge
...
* Splitting the library representation on disk in two.Gravatar Pierre-Marie Pédrot2015-06-24
* Disable precompilation for native_compute by default.Gravatar Guillaume Melquiond2015-05-14
* Remove almost all the uses of string concatenation when building error messages.Gravatar Guillaume Melquiond2015-04-23
* Extra fix to 934761875 and f4ee7ee31e4 on optimizing Import of severalGravatar Hugo Herbelin2015-04-17
* From X Require Y looks for X with absolute path, disregarding -R.Gravatar Pierre-Marie Pédrot2015-04-01
* Removing a probably incorrect on-the-fly require in a tactic.Gravatar Pierre-Marie Pédrot2015-04-01
* Dedicated type for on-demand objects in Library.Gravatar Pierre-Marie Pédrot2015-03-23
* Removing the whole library content from the summary.Gravatar Pierre-Marie Pédrot2015-03-16
* More invariants in Library.Gravatar Pierre-Marie Pédrot2015-03-16
* admit: replaced by give_up + Admitted (no proof_admitted : False, close #4032)Gravatar Enrico Tassi2015-03-11
* Fixing 934761875 about optimizing Import of several libraries at once (thanks...Gravatar Hugo Herbelin2015-02-23
* Windows: open .vo files in binary modeGravatar Enrico Tassi2015-02-05
* Optimized Import/Export the same way as Require Import/Export wasGravatar Hugo Herbelin2015-02-04
* Removing dead code.Gravatar Pierre-Marie Pédrot2015-02-02
* Remove dead code.Gravatar Maxime Dénès2015-01-17
* Partially revert "Forbid Require inside interactive modules and module types."Gravatar Maxime Dénès2015-01-17
* Avoid compilation warning... might not be the best fix though.Gravatar Matthieu Sozeau2015-01-17
* Made -print-mod-uid more silent and robust.Gravatar Maxime Dénès2015-01-13
* fixup to vi -> vio renamingGravatar Enrico Tassi2015-01-12
* Update headers.Gravatar Maxime Dénès2015-01-12
* Forbid Require inside interactive modules and module types.Gravatar Maxime Dénès2014-12-25
* Getting rid of Exninfo hacks.Gravatar Pierre-Marie Pédrot2014-12-16
* Fix for #3154: use CUnix.sys_command to call native compiler.Gravatar Maxime Dénès2014-12-16
* When loading libraries, feed back dependencies.Gravatar Carst Tankink2014-10-13
* STM: primitives to snapshot a .vi while in interactive modeGravatar Enrico Tassi2014-10-13
* library/opaqueTables: enable their use in interactive modeGravatar Enrico Tassi2014-10-13
* Removing dead code relative to the XML plugin.Gravatar Pierre-Marie Pédrot2014-09-08
* Feedback: LoadedFile + GoalsGravatar Enrico Tassi2014-07-11
* Checking that a library name is valid before compilation.Gravatar Pierre-Marie Pédrot2014-06-16
* Deprecate options -dont, -lazy, -force-load-proofs.Gravatar Guillaume Melquiond2014-06-13
* Fix native_compute for systems with a limited size for the command line.Gravatar Guillaume Melquiond2014-05-22
* Eliminating a potentially quadratic behaviour in Require, by using mapsGravatar Pierre-Marie Pédrot2014-05-11
* - Fix bug preventing apply from unfolding Fixpoints.Gravatar Matthieu Sozeau2014-05-06
* Adapt universe polymorphic branch to new handling of futures for delayed proofs.Gravatar Matthieu Sozeau2014-05-06
* Native compiler: hide compiled files in a .coq-native subdirectory.Gravatar Maxime Dénès2014-04-29
* STM: make -async-proofs on work from coqc tooGravatar Enrico Tassi2014-03-18
* vi2vo: universes handling finally fixedGravatar Enrico Tassi2014-03-11
* Fix lookup of native files when option -R is missing.Gravatar Guillaume Melquiond2014-03-07
* Library: when compiling multiple files, reset the opaque tablesGravatar Enrico Tassi2014-02-26
* Lazyconstr -> OpaqueproofGravatar Enrico Tassi2014-02-26
* New compilation mode -vi2voGravatar Enrico Tassi2014-02-26
* coqtop: -check-vi-tasks and -schedule-vi-checkingGravatar Enrico Tassi2014-01-05
* .vi files: .vo files without proofsGravatar Enrico Tassi2014-01-04
* Print logical name rather than path (thus allowing reproducible tests).Gravatar xclerc2013-12-02
* Native compiler: library compilation errors are now non fatal.Gravatar mdenes2013-10-28
* More monomorphic List.mem + List.assoc + ...Gravatar letouzey2013-10-24
* Turn many List.assoc into List.assoc_fGravatar letouzey2013-10-24
* Removing a bunch of generic equalities.Gravatar ppedrot2013-09-27
* Get rid of the uses of deprecated OCaml elements (still remaining compatible ...Gravatar xclerc2013-09-19
* Change in vo format : digest aren't Marshalled anymoreGravatar letouzey2013-08-22