index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
theories
/
Classes
/
EquivDec.v
Commit message (
Expand
)
Author
Age
*
This commit adds full universe polymorphism and fast projections to Coq.
Matthieu Sozeau
2014-05-06
*
Updating headers.
herbelin
2012-08-08
*
Open Local Scope ---> Local Open Scope, same with Notation and alii
letouzey
2012-07-05
*
Fixing tauto "special" behavior on singleton types w/ 2 parameters (bug #2680).
herbelin
2012-04-15
*
Final part of moving Program code inside the main code. Adapted add_definitio...
msozeau
2012-03-14
*
Everything compiles again.
msozeau
2012-03-14
*
Updated all headers for 8.3 and trunk
herbelin
2010-07-24
*
Remove the svn-specific $Id$ annotations
letouzey
2010-04-29
*
Remove various useless {struct} annotations
letouzey
2009-11-02
*
Add a new vernacular command for controling implicit generalization of
msozeau
2009-10-27
*
Fix the stdlib doc compilation + switch all .v file to utf8
letouzey
2009-09-28
*
Delete trailing whitespaces in all *.{v,ml*} files
glondu
2009-09-17
*
Fix compilation errors due to last commit.
msozeau
2009-09-15
*
Stop using a "Manual Implicit Arguments" flag and support them as soon
msozeau
2009-05-27
*
Just export RelationClasses for [Equivalence] through Setoid.
msozeau
2009-04-18
*
Rewrite of Program Fixpoint to overcome the previous limitations:
msozeau
2009-03-28
*
Last changes in type class syntax:
msozeau
2009-01-18
*
Move FunctionalExtensionality to Logic/ (someone please check that the
msozeau
2008-12-16
*
Generalized binding syntax overhaul: only two new binders: `() and `{},
msozeau
2008-12-14
*
Rename obligations_tactic to obligation_tactic and fix bugs #1893.
msozeau
2008-06-22
*
- Cleanup parsing of binders, reducing to a single production for all
msozeau
2008-05-11
*
Postpone the search for the recursive argument index from the user given
msozeau
2008-05-06
*
Fix the last compilation problem
msozeau
2008-04-09
*
Ajout des propriétés $Id:$ là où elles n'existaient pas ou n'étaient
herbelin
2008-04-01
*
- Second pass on implementation of let pattern. Parse "let ' par [as x]?
msozeau
2008-03-28
*
Various fixes on typeclasses:
msozeau
2008-03-27