| Commit message (Expand) | Author | Age |
* | Min, Max: for avoiding inelegant NPeano.max printing, we Export this lib | letouzey | 2010-02-10 |
* | Euclidean division for NArith | letouzey | 2010-02-10 |
* | Numbers: properties of min/max with respect to 0,S,P,add,sub,mul | letouzey | 2010-02-09 |
* | NPeano improved, subsumes NatOrderedType | letouzey | 2010-02-09 |
* | NSub: a missing lemma (sub usually decreases) | letouzey | 2010-02-09 |
* | NBinary improved, contains more, subsumes NOrderedType | letouzey | 2010-02-09 |
* | ZBinary (impl of Numbers via Z) reworked, comes earlier, subsumes ZOrderedType | letouzey | 2010-02-09 |
* | DoubleCyclic + NMake : typeclasses, more genericity, less ML macro-generation | letouzey | 2010-02-08 |
* | Division in numbers: kills some Include to avoid bad alias Zsucc = ZDiv.Z.Z'.S | letouzey | 2010-01-29 |
* | NMake (and hence BigN): shiftr, shiftl now in the signature NSig | letouzey | 2010-01-25 |
* | NMake: several things need not be macro-generated | letouzey | 2010-01-25 |
* | Ring31 : a ring structure and tactic for int31 | letouzey | 2010-01-19 |
* | NMake_gen: fix previous commit (some spaces were critical), remove some more ... | letouzey | 2010-01-19 |
* | NMake_gen: no more spaces at end of lines | letouzey | 2010-01-19 |
* | More improvements of BigN, BigZ, BigQ: | letouzey | 2010-01-18 |
* | BigN, BigZ, BigQ: presentation via unique module with both ops and props | letouzey | 2010-01-17 |
* | Simplification of OrdersTac thanks to the functor application ! with no inline | letouzey | 2010-01-17 |
* | Avoid some more re-declarations of Equivalence instances | letouzey | 2010-01-14 |
* | Numbers/.../NDefOps: one more property about ltb | letouzey | 2010-01-12 |
* | Numbers: some more proofs about sub,add,le,lt for natural numbers | letouzey | 2010-01-12 |
* | Numbers: two more Local Obligation Tactic | letouzey | 2010-01-12 |
* | Support "Local Obligation Tactic" (now the default in sections). | msozeau | 2010-01-11 |
* | Numbers: BigN and BigZ get instantiations of all properties about div and mod | letouzey | 2010-01-08 |
* | Numbers: axiomatization + generic properties of abs and sgn. | letouzey | 2010-01-08 |
* | NZAxioms plus a compare allows to build an OrderedType | letouzey | 2010-01-08 |
* | Nicer names: DecidableType2* --> Equalities*, OrderedType2* --> Orders* | letouzey | 2010-01-07 |
* | Include can accept both Module and Module Type | letouzey | 2010-01-07 |
* | Numbers: separation of funs, notations, axioms. Notations via module, without... | letouzey | 2010-01-07 |
* | Patch on subtyping check of opaque constants. | soubiran | 2010-01-06 |
* | "by" becomes officially a reserved keyword of Coq (fixes "rewrite ... at ... ... | letouzey | 2010-01-06 |
* | Numbers abstract layer: more Module Type, used especially for divisions. | letouzey | 2010-01-05 |
* | Avoid declaring hints about refl/sym/trans of eq in DecidableType2 | letouzey | 2010-01-05 |
* | Division in Numbers: proofs with less auto (less sensitive to hints, in parti... | letouzey | 2010-01-05 |
* | Division in Numbers: factorisation of signatures | letouzey | 2010-01-05 |
* | Specific syntax for Instances in Module Type: Declare Instance | letouzey | 2010-01-04 |
* | RelationPairs: stop loading it in all Numbers, stop maximal args with fst/snd | letouzey | 2009-12-18 |
* | Division in Numbers : more properties, new filenames based on a paper by R. B... | letouzey | 2009-12-17 |
* | Division in Numbers: more properties proved (still W.I.P.) | letouzey | 2009-12-16 |
* | A generic euclidean division in Numbers (Still Work-In-Progress) | letouzey | 2009-12-15 |
* | NZDomain: investigation of the shape of NZ domain, more results about ofnat:n... | letouzey | 2009-12-10 |
* | Factorisation between Makefile and ocamlbuild systems : .vo to compile are in... | letouzey | 2009-12-09 |
* | Forgot a file in last commit. | msozeau | 2009-12-06 |
* | Fix anomaly when using typeclass resolution with filtered hyps in evars. | msozeau | 2009-12-06 |
* | Fix backtracking heuristic in typeclass resolution. | msozeau | 2009-11-30 |
* | Diamond-shape instead of linear hiearchy in Numbers/NatInt | letouzey | 2009-11-18 |
* | New syntax <+ for chains of Include (or Include Type) (or Include Self (Type)) | letouzey | 2009-11-16 |
* | Taking advantage of the new "Include Self Type" in DecidableType2 and NZAxioms | letouzey | 2009-11-16 |
* | BigQ / BigN / BigZ syntax and scope improvements (sequel to 12504) | letouzey | 2009-11-12 |
* | Repair interpretation of numeral for BigQ, add a printer (close #2160) | letouzey | 2009-11-12 |
* | SpecViaZ.NSig: all-in-one spec for [pred] and [sub] based on ZMax | letouzey | 2009-11-10 |