index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
toplevel
Commit message (
Expand
)
Author
Age
*
Inclusion of functors with restricted signature is now forbidden (fix #3746)
Pierre Letouzey
2015-12-22
*
Flag -compat 8.4 now loads Coq.Compat.Coq84.
Maxime Dénès
2015-12-14
*
Print Assumptions: improve detection of case on an axiom of False
Enrico Tassi
2015-12-09
*
Univs/Program: update the universe context with global universe
Matthieu Sozeau
2015-12-02
*
Fix bug #4444: Next Obligation performed after a Section opening was
Matthieu Sozeau
2015-12-02
*
Univs: correctly register universe binders for lemmas.
Matthieu Sozeau
2015-11-28
*
Fix [Polymorphic Hint Rewrite].
Matthieu Sozeau
2015-11-27
*
Univs: carry on universe substitution when defining obligations of
Matthieu Sozeau
2015-11-24
*
Fix output of universe arcs. (Fix bug #4422)
Guillaume Melquiond
2015-11-23
*
Univs: generation of induction schemes should not generated useless
Matthieu Sozeau
2015-11-20
*
Allow program hooks to see the refined universe_context at the end of a
Matthieu Sozeau
2015-11-19
*
Adding syntax "Show id" to show goal named id (shelved or not).
Hugo Herbelin
2015-11-02
*
Command.declare_definition: grab the fix_exn early (follows 77cf18e)
Enrico Tassi
2015-10-30
*
Add a way to get the right fix_exn in external vernacular commands
Matthieu Sozeau
2015-10-30
*
Accept option -compat 8.5. (Fix bug #4393)
Guillaume Melquiond
2015-10-29
*
Univs: local names handling.
Matthieu Sozeau
2015-10-28
*
Avoid type checking private_constants (side_eff) again during Qed (#4357).
Enrico Tassi
2015-10-28
*
Univs: fix bug #4375, accept universe binders on (co)-fixpoints
Matthieu Sozeau
2015-10-28
*
Fix bugs 4389, 4390 and 4391 due to wrong handling of universe names
Matthieu Sozeau
2015-10-27
*
Minor module cleanup : error HigherOrderInclude was never happening
Pierre Letouzey
2015-10-25
*
Miscellaneous typos, spacing, US spelling in comments or variable names.
Hugo Herbelin
2015-10-18
*
Lemmas accept the Local flag.
Pierre-Marie Pédrot
2015-10-17
*
Remove -vm flag of coqtop.
Maxime Dénès
2015-10-14
*
Fixing bug #4367: Wrong error message in unification.
Pierre-Marie Pédrot
2015-10-14
*
Fix some typos.
Guillaume Melquiond
2015-10-13
*
Fix Definition id := Eval <redexpr> in by passing the right universe
Matthieu Sozeau
2015-10-12
*
Code cleaning in VM (with Benjamin).
Maxime Dénès
2015-10-09
*
Fix Next Obligation to not raise an anomaly in case of mutual
Matthieu Sozeau
2015-10-09
*
Axioms now support the universe binding syntax.
Pierre-Marie Pédrot
2015-10-08
*
aux_file: export API to ease writing of a Proof Using annotator.
Enrico Tassi
2015-10-08
*
Proof using: let-in policy, optional auto-clear, forward closure*
Enrico Tassi
2015-10-08
*
Spawn: use each socket exclusively for writing or reading
Enrico Tassi
2015-10-08
*
Goptions: new value type: optional string
Enrico Tassi
2015-10-08
*
Univs: fix FingerTree contrib.
Matthieu Sozeau
2015-10-07
*
Univs: add Strict Universe Declaration option (on by default)
Matthieu Sozeau
2015-10-07
*
Univs: fix handling of evar_map in identity coercion construction.
Matthieu Sozeau
2015-10-05
*
Fix after rebase...
Matthieu Sozeau
2015-10-02
*
Univs: fix inference of the lowest sort for records.
Matthieu Sozeau
2015-10-02
*
Univs: correcly compute the levels of records when they fall in Prop.
Matthieu Sozeau
2015-10-02
*
Univs/program: handle side effects in obligations.
Matthieu Sozeau
2015-10-02
*
Univs: fix Show Universes.
Matthieu Sozeau
2015-10-02
*
Univs: fix environment handling in scheme building.
Matthieu Sozeau
2015-10-02
*
Univs: fix after rebase (from_ctx/from_env)
Matthieu Sozeau
2015-10-02
*
Univs: fix many evar_map initializations and leaks.
Matthieu Sozeau
2015-10-02
*
Universes: enforce Set <= i for all Type occurrences.
Matthieu Sozeau
2015-10-02
*
Prevent States.intern_state and System.extern_intern from looking up files in...
Guillaume Melquiond
2015-09-29
*
Remove some uses of Loadpath.get_paths.
Guillaume Melquiond
2015-09-29
*
Make -load-vernac-object respect the loadpath.
Guillaume Melquiond
2015-09-28
*
The -require option now accepts a logical path instead of a physical one.
Pierre-Marie Pédrot
2015-09-25
*
Updating the documentation and the toolchain w.r.t. the change in -compile.
Pierre-Marie Pédrot
2015-09-25
[next]