index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
parsing
/
g_vernac.ml4
Commit message (
Expand
)
Author
Age
*
Added support for definition of fixpoints using tactics.
herbelin
2009-11-27
*
Module subtyping : allow many <: and module type declaration with <:
letouzey
2009-11-18
*
New syntax <+ for chains of Include (or Include Type) (or Include Self (Type))
letouzey
2009-11-16
*
Include Self (Type) Foo: applying a (Type) Functor to the current context
letouzey
2009-11-16
*
Document Generalizable Variables, and change syntax to
msozeau
2009-11-15
*
Added support for multiple where-clauses in Inductive and co (see wish #2163).
herbelin
2009-11-11
*
Misc fixes.
msozeau
2009-11-06
*
Integrate a few improvements on typeclasses and Program from the equations br...
msozeau
2009-10-28
*
Module type expressions of the form (Fsig X) with Definition foo := bar are n...
soubiran
2009-10-28
*
Add a new vernacular command for controling implicit generalization of
msozeau
2009-10-27
*
New cleaning phase of the Local/Global option management
herbelin
2009-10-26
*
Improved the treatment of Local/Global options (noneffective Local on
herbelin
2009-10-25
*
Add support for Local Declare ML Module
glondu
2009-09-29
*
Delete trailing whitespaces in all *.{v,ml*} files
glondu
2009-09-17
*
- Addition of "Reserved Infix" continued.
herbelin
2009-09-14
*
- Inductive types in the "using" option of auto/eauto/firstorder are
herbelin
2009-09-13
*
Generalized the possibility to refer to a global name by a notation
herbelin
2009-09-11
*
Postpone checking of Local/Global to allow grammar extensions to use it
msozeau
2009-09-02
*
Ajout de la gestion de Local et Global pour les options (au sens de
aspiwack
2009-08-14
*
Add support for "Infix ... := constr" instead of just "Infix ... := ref".
herbelin
2009-08-11
*
Improved parameterization of Coq:
herbelin
2009-08-02
*
- Granted wish #2138 (support for local binders in syntax of Record fields).
herbelin
2009-07-15
*
Allow anonymous instances again, with syntax [Instance: T] where T
msozeau
2009-06-15
*
- Cleaning (unification of ML names, removal of obsolete code,
herbelin
2009-04-27
*
Some dead code removal + cleanups
letouzey
2009-04-08
*
Optionally list opaque constants in addition to axions/variables in
msozeau
2009-03-09
*
commande Timeout + compaction des traces de debug_tactic
barras
2009-03-04
*
Do not reserve the keyword "Infer".
puech
2009-02-03
*
Les records déclarés avec Record ne peuvent plus être récursifs (le
aspiwack
2009-01-19
*
- Structuring Numbers and fixing Setoid in stdlib's doc.
herbelin
2009-01-19
*
Last changes in type class syntax:
msozeau
2009-01-18
*
DISCLAIMER
puech
2009-01-17
*
Fixing/improving management of uniform prefix Local and Global
herbelin
2009-01-14
*
- Standardized prefix use of "Local"/"Global" modifiers as decided in
herbelin
2009-01-13
*
- Added support for subterm matching in SearchAbout.
herbelin
2008-12-29
*
- coq_makefile: target install now respects the original tree structure
herbelin
2008-12-24
*
Generalized binding syntax overhaul: only two new binders: `() and `{},
msozeau
2008-12-14
*
Fix mixup between Record, Structure and Class by adding a new variant for
msozeau
2008-11-10
*
More factorization of inductive/record and typeclasses: move class
msozeau
2008-11-09
*
Move Record desugaring to constrintern and add ability to use notations
msozeau
2008-11-05
*
Nouvelle syntaxe pour écrire des records (co)inductifs :
aspiwack
2008-11-05
*
Renommage "Global Instance" en "Instance Global" pour uniformisation
herbelin
2008-10-20
*
- Export de pattern_ident vers les ARGUMENT EXTEND and co.
herbelin
2008-10-19
*
Backporting 11445 from 8.2 to trunk (negative conditions in
herbelin
2008-10-11
*
Correct handling of implicit arguments in [Equations] definitions,
msozeau
2008-09-03
*
Uniformisation du format des messages d'erreur (commencent par une
herbelin
2008-07-17
*
- Improve [Context] vernacular to allow arbitrary binders, not just
msozeau
2008-07-07
*
- Correction de la version simplifiée (filtrage sur deux sig
herbelin
2008-06-09
*
Improvements on coqdoc by adding more information into .glob
msozeau
2008-05-30
*
Strategy commands are now exported
barras
2008-05-22
[next]