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