index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
theories
/
NArith
/
BinNat.v
Commit message (
Expand
)
Author
Age
*
DecidableType: A specification via boolean equality as an alternative to eq_dec
letouzey
2009-11-10
*
Better visibility of the inductive CompSpec used to specify comparison functions
letouzey
2009-11-03
*
OrderedType implementation for various numerical datatypes + min/max structures
letouzey
2009-11-03
*
Delete trailing whitespaces in all *.{v,ml*} files
glondu
2009-09-17
*
OrderedTypeEx.N_as_OT use Nlt, various minor improvements in N/ZArith
letouzey
2009-07-24
*
- Another bug in get_sort_family_of (sort-polymorphism of constants and
herbelin
2008-12-28
*
Definition of N moves back to BinNat (partial backtrack of commits 10298-10300)
letouzey
2008-04-16
*
Proposal of a nice notation for constructors xI and xO of type positive
letouzey
2008-02-10
*
Moved several lemmas from theories/Numbers/NumPrelude to theories/Init/Logic.
emakarov
2007-11-08
*
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10300 85f007b7-540e-0...
emakarov
2007-11-07
*
Forgot a backslash in Makefile.common. Added "(only parsing)" in BinNat.v.
emakarov
2007-11-07
*
Replaced BinNat with a new version that is based on theories/Numbers/Natural/...
emakarov
2007-11-07
*
Added the compilation of theories/Numbers to Makefile.common. The following t...
emakarov
2007-10-01
*
Changed the definition of Nminus in BinNat.v by removing comparison.
emakarov
2007-09-20
*
Extension of NArith: Nminus, Nmin, etc
letouzey
2007-06-07
*
Added the following theorems to BinPos:
emakarov
2007-03-30
*
qq proprietes de plus sur Ncompare
letouzey
2006-04-29
*
Un gros coup de lifting pour IntMap:
letouzey
2006-04-25
*
ouverture du bon scope (positive_scope) derriere le constructeur Npos de N
letouzey
2006-04-06
*
Changement dans les boxed values .
gregoire
2004-11-12
*
Nouvelle en-tête
herbelin
2004-07-16
*
Remplacement des fichiers .v ancienne syntaxe de theories, contrib et states ...
herbelin
2003-11-29
*
ajout Pnat (suite)
herbelin
2003-11-21
*
Extraction des lemmes sur convert/nat_of_P de BinPos vers Pnat; ajout Pcase e...
herbelin
2003-11-21
*
Ordre standard pour l'associativite
herbelin
2003-11-14
*
Noms/énoncés plus canoniques
herbelin
2003-11-12
*
Notations
herbelin
2003-11-05
*
Ajout répertoire NArith pour l'arithmétique binaire sur les nombres positif...
herbelin
2003-11-05