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