aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
Commit message (Expand)AuthorAge
* SearchAbout and similar: add a customizable blacklistGravatar letouzey2011-08-11
* Take benefit of bullets available by default in PreludeGravatar herbelin2011-08-10
* Less ambitious application of a notation for eq_rect. We proposedGravatar herbelin2011-08-10
* Moved the declaration of "Classic" being the default proof mode to coqtop.ml ...Gravatar aspiwack2011-08-09
* New proposition "rewrite Heq in H" for eq_rect (assuming that there isGravatar herbelin2011-08-08
* All the parameters of or can be implicits.Gravatar pboutill2011-07-26
* Same Implicit Arguments rule for sumbool and sumor.Gravatar pboutill2011-07-26
* Tentative abbreviation "rew Heq in H" for eq_rect. (feedback welcome)Gravatar herbelin2011-07-16
* Added a characterization of unique existence.Gravatar herbelin2011-07-16
* Arithemtic: more concerning compare, eqb, leb, ltbGravatar letouzey2011-06-20
* Some simplifications in NZDomainGravatar letouzey2011-06-20
* Wf.iter_nat becomes Peano.nat_iter (with an implicit arg)Gravatar letouzey2011-05-05
* Modularization of BinNat + fixes of stdlibGravatar letouzey2011-05-05
* Better comments and organisation in Datatypes.vGravatar letouzey2011-05-05
* Fixing an "apply -> ... in hyp" bug (the hyp was considered as a fixedGravatar herbelin2011-04-28
* Init: some results in Type should rather be Defined than QedGravatar letouzey2011-03-21
* CompareSpec: a slight generalization/reformulation of CompSpecGravatar letouzey2011-03-17
* Remove the "Boxed" syntaxes and the const_entry_boxed fieldGravatar letouzey2011-01-28
* First release of Vector library.Gravatar pboutill2010-12-10
* Used multiple lists of implicit arguments to transfer the choices ofGravatar herbelin2010-10-23
* Using multiple lists of implicit arguments in Program for preservingGravatar herbelin2010-10-03
* Updated all headers for 8.3 and trunkGravatar herbelin2010-07-24
* Made notations for exists, exists! and notations of Utf8.v recursive notationsGravatar herbelin2010-07-22
* Bool: shorter and more systematic proofs + an iff lemma about eqbGravatar letouzey2010-07-16
* Bool: iff lemmas about or, a reflect inductive, an is_true functionGravatar letouzey2010-07-10
* clear/revert dependent: restrict to hyp(h) instead of ident(h)Gravatar letouzey2010-06-18
* New tactic "clear dependent", for the moment in ltac in Init/TacticsGravatar letouzey2010-06-17
* Remove the svn-specific $Id$ annotationsGravatar letouzey2010-04-29
* Here comes the commit, announced long ago, of the new tactic engine.Gravatar aspiwack2010-04-22
* Arith's min and max placed in Peano (+basic specs max_l and co)Gravatar letouzey2010-02-17
* CompSpec2Type is used to build functions, it should be Defined, not QedGravatar letouzey2010-02-13
* CompSpecType, a clone of CompSpec but in Type instead of PropGravatar letouzey2010-02-12
* Init/Logic: commutativity and associativity of /\ and \/Gravatar letouzey2010-01-08
* Factorisation between Makefile and ocamlbuild systems : .vo to compile are in...Gravatar letouzey2009-12-09
* Some lemmas about dependent choice + extensions of Compare_dec +Gravatar herbelin2009-11-16
* Datatypes.length and app defined back via fun+fix instead of FixpointGravatar letouzey2009-11-06
* Better visibility of the inductive CompSpec used to specify comparison functionsGravatar letouzey2009-11-03
* Remove various useless {struct} annotationsGravatar letouzey2009-11-02
* list, length, app are migrated from List to DatatypesGravatar letouzey2009-11-02
* Init/Tactics.v: tactic with nicer name 'exfalso' for 'elimtype False'Gravatar letouzey2009-10-08
* Implicit argument of Logic.eq become maximally insertedGravatar letouzey2009-10-08
* Delete trailing whitespaces in all *.{v,ml*} filesGravatar glondu2009-09-17
* New tactic to rewrite decidability lemmas when one knows which sideGravatar herbelin2009-08-24
* Fixed extra space in printing notation { x & P } + minor other thingsGravatar herbelin2009-08-11
* OrderedTypeEx.N_as_OT use Nlt, various minor improvements in N/ZArithGravatar letouzey2009-07-24
* Miscellaneous practical commits: Gravatar herbelin2009-06-29
* Parsing files for numerals (+ ascii/string) moved into pluginsGravatar letouzey2009-03-27
* Better mechanism for loading initial pluginsGravatar letouzey2009-03-14
* - Temptative change to notations like "as [|n H]_eqn" or "as [|n H]_eqn:H",Gravatar herbelin2009-01-02
* Switched to "standardized" names for the properties of eq andGravatar herbelin2009-01-01