aboutsummaryrefslogtreecommitdiffhomepage
path: root/library
Commit message (Collapse)AuthorAge
...
* | Make -load-vernac-object respect the loadpath.Gravatar Guillaume Melquiond2015-09-28
| | | | | | | | | | | | | | | | | | | | This command-line option was behaving like the old -require, except that it did not do Import. In other words, it was loading files without respecting the loadpath. Now it behaves exactly like Require, while -require now behaves like Require Import. This patch also removes Library.require_library_from_file and all its dependencies, since they are no longer used inside Coq.
| * Show assumptions of well-foundedness in `Print Assumptions`Gravatar Arnaud Spiwack2015-09-25
| |
* | The -require option now accepts a logical path instead of a physical one.Gravatar Pierre-Marie Pédrot2015-09-25
| |
* | The -compile option now accepts ".v" files and outputs a warning otherwise.Gravatar Pierre-Marie Pédrot2015-09-25
| |
| * Propagate `Guarded` flag from syntax to kernel.Gravatar Arnaud Spiwack2015-09-25
| | | | | | | | The path is quite a bit of a maze, this commit is not as simple as it ought to be. Something more robust than a boolean should be used here.
* | Hopefully better names to constructors of internal_flag, as discussedGravatar Hugo Herbelin2015-09-23
| | | | | | | | with Enrico.
* | Nametab: print debug notice only in debug mode.Gravatar Maxime Dénès2015-09-20
| |
* | Add an if_verbose for "Fetching opaque proofs ..."Gravatar mlasson2015-09-03
| | | | | | | | | | I do not think that this information is worth displaying without the verbose flag.
* | Fixing anomaly #3743 while printing an error message involving evar constraints.Gravatar Hugo Herbelin2015-07-16
| | | | | | | | | | | | | | | | Indeed, the name of a bound variable was lost when unifying under a Prod in evarconv. The error message for "Unable to satisfy the following constraints" is still to be improved though.
* | Option -type-in-type: added support in checker and making it contaminatingGravatar Hugo Herbelin2015-07-10
| | | | | | | | | | | | | | | | | | | | in vo files (this was not done yet in 24d0027f0 and 090fffa57b). Reused field "engagement" to carry information about both impredicativity of set and type in type. For the record: maybe some further checks to do around the sort of the inductive types in coqchk?
* | Native compiler: refactor code handling pre-computed values.Gravatar Maxime Dénès2015-07-10
| | | | | | | | Fixes #4139 (Not_found exception with Require in modules).
* | Improve semantics of -native-compiler flag.Gravatar Maxime Dénès2015-07-09
| | | | | | | | | | | | | | | | | | | | Since Guillaume's, launching coqtop without -native-compiler and call native_compute would mean recompiling silently all dependencies, even if they had been precompiled (e.g. the stdlib). The new semantics is that -native-compiler disables separate compilation of the current library, but still tries to load precompiled dependencies. If loading fails when the flag is on, coqtop stays silent.
* | Univs/minimization: Fix unused variable bug.Gravatar Matthieu Sozeau2015-07-07
| |
* | Assumptions: more informative print for False axiom (Close: #4054)Gravatar Enrico Tassi2015-06-29
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | When an axiom of an empty type is matched in order to inhabit a type, do print that type (as if each use of that axiom was a distinct foo_subproof). E.g. Lemma w : True. Proof. case demon. Qed. Lemma x y : y = 0 /\ True /\ forall w, w = y. Proof. split. case demon. split; [ exact w | case demon ]. Qed. Print Assumptions x. Prints: Axioms: demon : False used in x to prove: forall w : nat, w = y used in w to prove: True used in x to prove: y = 0
* | Fix bug #4254 with the help of J.H. JourdanGravatar Matthieu Sozeau2015-06-26
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | 1) We now _assign_ the smallest possible arities to mutual inductive types and eventually add leq constraints on the user given arities. Remove useless limitation on instantiating algebraic universe variables with their least upper bound if they have upper constraints as well. 2) Do not remove non-recursive variables when computing minimal levels of inductives. 3) Avoid modifying user-given arities if not necessary to compute the minimal level of an inductive. 4) We correctly solve the recursive equations taking into account the user-declared level.
* | Wrapped the declare_object function to pretty-print anomalies at loading time.Gravatar Thomas Sibut-Pinote2015-06-25
| |
| * Make inductives that were assumed positive appear in `Print Assumptions`.Gravatar Arnaud Spiwack2015-06-24
| | | | | | | | They appear as axioms of the form `Foo is positive`.
| * Add a corresponding field in `mutual_inductive_entry` (part 1).Gravatar Arnaud Spiwack2015-06-24
| | | | | | | | The field in `mutual_inductive_entry` requires that a mutually inductive definition be checked or not, whereas the field in `mutual_inductive_body` asserts that it has or has not been.
| * Merge branch 'v8.5'Gravatar Pierre-Marie Pédrot2015-06-24
| |\ | |/ |/|
* | On-demand Require.Gravatar Pierre-Marie Pédrot2015-06-24
| | | | | | | | | | | | Marshalled libraries are only loaded when needed and dropped thereafter. This might be costly for Require inside modules, but such a practice is discouraged anyway.
* | Splitting the library representation on disk in two.Gravatar Pierre-Marie Pédrot2015-06-24
| | | | | | | | | | The first part only contains the summary of the library, while the second one contains the effective content of it.
| * Wrapped the declare_object function to pretty-print anomalies at loading time.Gravatar Thomas Sibut-Pinote2015-06-23
|/
* Fix bug #3446.Gravatar Matthieu Sozeau2015-06-11
| | | | Wrong handling of algebraic universes that have upper bounds.
* Fix bug #4159Gravatar Matthieu Sozeau2015-05-27
| | | | | | Some asynchronous constraints between initial universes and the ones at the end of a proof were forgotten. Also add a message to print universes indicating if all the constraints are processed already or not.
* Disable precompilation for native_compute by default.Gravatar Guillaume Melquiond2015-05-14
| | | | | | | | | | | | | | Note that this does not prevent using native_compute, but it will force on-the-fly recompilation of dependencies whenever it is used. Precompilation is enabled for the standard library, assuming native compilation was enabled at configuration time. If native compilation was disabled at configuration time, native_compute falls back to vm_compute. Failure to precompile is a hard error, since it is now explicitly required by the user.
* Remove almost all the uses of string concatenation when building error messages.Gravatar Guillaume Melquiond2015-04-23
| | | | | | Since error messages are ultimately passed to Format, which has its own buffers for concatenating strings, using concatenation for preparing error messages just doubles the workload and increases memory pressure.
* Tactical `progress` compares term up to potentially equalisable universes.Gravatar Arnaud Spiwack2015-04-22
| | | | | Followup of: f7b29094fe7cc13ea475447bd30d9a8b942f0fef . In particular, re-closes #3593. As a side effect, fixes an undiscovered bug of the `eq_constr` tactic which didn't consider terms up to evar instantiation.
* Extra fix to 934761875 and f4ee7ee31e4 on optimizing Import of severalGravatar Hugo Herbelin2015-04-17
| | | | libraries at once (see #4193).
* Strengthen minimization: it shouldn't set a universe u to a max if itGravatar Matthieu Sozeau2015-04-09
| | | | has a strict upper bound.
* Make it possible for -R to override the existing implicit setting of a path.Gravatar Guillaume Melquiond2015-04-02
| | | | | Without this commit, passing "-R theories Coq" to "coqtop -nois" has no effect since "-Q theories Coq" has already been done implicitly.
* 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
| | | | | Also removed the require function it was using, as it is absent from the remaining of the code.
* Removing the unused root flag from loadpaths.Gravatar Pierre-Marie Pédrot2015-03-31
|
* A more reasonable implementation of Loadpath.Gravatar Pierre-Marie Pédrot2015-03-31
| | | | | | | | The new behaviour is simple: either a path is in the loadpaths or it is not. No more wild expansions of paths! This should not affect -R and -Q, but it does change the semantics of -I -as. Still, there are no more users of it and it only does so in a subtle way.
* Summary: fix code to detect functional values in summaryGravatar Enrico Tassi2015-03-25
|
* 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
| | | | It is still present in the libstack, though.
* More invariants in Library.Gravatar Pierre-Marie Pédrot2015-03-16
| | | | | We explicit the fact that we only need the name of the library in most of the summaries.
* admit: replaced by give_up + Admitted (no proof_admitted : False, close #4032)Gravatar Enrico Tassi2015-03-11
| | | | | | | | | | | | | | | - no more inconsistent Axiom in the Prelude - STM can now process Admitted proofs asynchronously - the quick chain can stock "Admitted" jobs in .vio files - the vio2vo step checks the jobs but does not stock the result in the opaque tables (they have no slot) - Admitted emits a warning if the proof is complete - Admitted uses the (partial) proof term to infer section variables used (if not given with Proof using), like for Qed - test-suite: extra line Require TestSuite.admit to each file making use of admit - test-suite/_CoqProject: to pass to CoqIDE and PG the right -Q flag to find TestSuite.admit
* STM: proof state also includes meta countersGravatar Enrico Tassi2015-02-25
| | | | | Workers send back incomplete system states (only the proof part). Such part must include the meta/evar counter.
* Refactoring in [Constr].Gravatar Arnaud Spiwack2015-02-24
| | | | [compare_head_gen] defined in terms of [compare_head_gen_leq]. Remove an unused argument from [compare_head_gen_leq].
* Fix some typos in comments.Gravatar Guillaume Melquiond2015-02-23
|
* Fixing 934761875 about optimizing Import of several libraries at once ↵Gravatar Hugo Herbelin2015-02-23
| | | | (thanks to Enrico for noticing a bug).
* Documenting the caveat of assumption printing in the mli.Gravatar Pierre-Marie Pédrot2015-02-21
|
* Tentative fix for bug #4078.Gravatar Pierre-Marie Pédrot2015-02-21
|
* More resilient implementation of Print Assumptions.Gravatar Pierre-Marie Pédrot2015-02-21
| | | | | | | | | Instead of registering all the transitive dependencies of a term in one go, we rather recursively build the graph of direct dependencies of this term. This is finer-grained and offers a better API. The traversal now uses the standard term fold operation, and also registers inductives and constructors encountered in the traversal.
* Deprecated options issue a warning.Gravatar Pierre-Marie Pédrot2015-02-17
|
* Fixing bug #4053.Gravatar Pierre-Marie Pédrot2015-02-17
|
* Better comment for [type_of_global_unsafe].Gravatar Matthieu Sozeau2015-02-16
|
* Comment on the unsafe_ functions in Global.Gravatar Matthieu Sozeau2015-02-16
|