index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
toplevel
/
command.ml
Age
Commit message (
Expand
)
Author
2015-10-30
Command.declare_definition: grab the fix_exn early (follows 77cf18e)
Enrico Tassi
2015-10-28
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-27
Fix bugs 4389, 4390 and 4391 due to wrong handling of universe names
Matthieu Sozeau
2015-10-12
Fix Definition id := Eval <redexpr> in by passing the right universe
Matthieu Sozeau
2015-10-08
Axioms now support the universe binding syntax.
Pierre-Marie Pédrot
2015-10-07
Univs: add Strict Universe Declaration option (on by default)
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-09-25
Declare assumptions of well-founded definitions as unsafe.
Arnaud Spiwack
2015-09-25
Propagate `Guarded` flag from syntax to kernel.
Arnaud Spiwack
2015-09-25
Add a flag in `VernacFixpoint` and `VernacCoFixpoint` to control assuming gua...
Arnaud Spiwack
2015-09-14
Univs: Add universe binding lists to definitions
Matthieu Sozeau
2015-07-10
Option -type-in-type: added support in checker and making it contaminating
Hugo Herbelin
2015-06-26
Fix bug #4254 with the help of J.H. Jourdan
Matthieu Sozeau
2015-06-26
Add a flag to deactivate guard checking in the kernel.
Arnaud Spiwack
2015-06-24
When assuming an inductive type positive, then it is declared "unsafe" to the...
Arnaud Spiwack
2015-06-24
Add corresponding field in `VernacInductive`.
Arnaud Spiwack
2015-06-24
Add a corresponding field in `mutual_inductive_entry` (part 1).
Arnaud Spiwack
2015-05-27
Fix bug #4159
Matthieu Sozeau
2015-05-13
Safer typing primitives.
Pierre-Marie Pédrot
2015-05-01
Fixing computation of implicit arguments by position in fixpoints (#4217).
Hugo Herbelin
2015-04-23
Remove almost all the uses of string concatenation when building error messages.
Guillaume Melquiond
2015-02-10
Fixing #4017, #3726 (use of implicit arguments was lost in multiple variable ...
Hugo Herbelin
2015-01-21
Add the possibility of defining opaque terms with program.
mlasson
2015-01-12
Update headers.
Maxime Dénès
2015-01-05
kernel/ind Change interface of declare_mind and declare_mutual
Matthieu Sozeau
2014-11-23
Pass around information on the use of template polymorphism for
Matthieu Sozeau
2014-10-25
This commit introduces changes in induction and destruct.
Hugo Herbelin
2014-10-24
Change reduction_of_red_expr to return an e_reduction_function returning
Matthieu Sozeau
2014-10-22
Lemmas/Pfedit: use full evar_map instead of universe contexts to start proofs.
Arnaud Spiwack
2014-10-03
Fixing #3193 (honoring implicit arguments in local definitions).
Hugo Herbelin
2014-09-30
Add syntax for naming new goals in refine: writing ?[id] instead of _
Hugo Herbelin
2014-09-13
Providing a -type-in-type option for collapsing the universe hierarchy.
Hugo Herbelin
2014-09-12
Uniformisation of the order of arguments env and sigma.
Hugo Herbelin
2014-09-12
Referring to evars by names. Added a parser for evars (but parsing of
Hugo Herbelin
2014-09-10
Fix categorization of recursive inductives.
Matthieu Sozeau
2014-09-08
Parsing of Type@{max(i,j)}.
Matthieu Sozeau
2014-09-07
Fixing bug #3492.
Pierre-Marie Pédrot
2014-09-04
Types declared as Variants really do not accept recursive definitions.
Arnaud Spiwack
2014-08-30
Simplify even further the declaration of primitive projections,
Matthieu Sozeau
2014-08-29
Fixing commit 50237af2.
Pierre-Marie Pédrot
2014-08-28
Fixing bug #3528.
Pierre-Marie Pédrot
2014-08-28
Change the way primitive projections are declared to the kernel.
Matthieu Sozeau
2014-07-25
- Do module substitution inside mind_record.
Matthieu Sozeau
2014-07-11
Properly add a Set lower bound on any polymorphic inductive in Type with
Matthieu Sozeau
2014-07-03
Cleanup code related to the constraint solving, which sits now outside the
Matthieu Sozeau
2014-07-03
Properly compute the transitive closure of the system of constraints
Matthieu Sozeau
2014-07-01
Add toplevel commands to declare global universes and constraints.
Matthieu Sozeau
[prev]
[next]