aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
Commit message (Expand)AuthorAge
* [Coercion]s use [Sortclass], not [Prop] (in docs)Gravatar Jason Gross2014-01-24
* Better unification for [projT1] and [proj1_sig].Gravatar Jason Gross2013-12-12
* Adding Acc_intro_generator in order to help computations of Function in parti...Gravatar forest2013-11-20
* Side effect free implementation of admit (Isabelle's oracle)Gravatar gareuselesinge2013-08-08
* Improving printing of 'rew' notationGravatar herbelin2013-05-05
* Relaxing the constraint on eta-expanding on the fly while looking forGravatar herbelin2013-05-05
* Added group properties of eq_refl, eq_sym, eq_transGravatar herbelin2013-04-17
* Unset Asymmetric PatternsGravatar pboutill2013-01-18
* nat_iter n f x -> nat_rect _ x (fun _ => f) nGravatar pboutill2012-12-21
* Some lemmas on property of rewriting. It will probably be worth atGravatar herbelin2012-11-15
* Change Hint Resolve, Immediate to take a global reference as argumentGravatar msozeau2012-10-26
* Removed a few calls to "Opaque" in Logic.v ineffective since at leastGravatar herbelin2012-10-24
* No more states/initial.coq, instead coqtop now requires Prelude.voGravatar letouzey2012-08-23
* Updating headers.Gravatar herbelin2012-08-08
* induction/destruct : nicer syntax for generating equations (solves #2741)Gravatar letouzey2012-07-09
* Kills the useless tactic annotations "in |- *"Gravatar letouzey2012-07-05
* ZArith + other : favor the use of modern names instead of compat notationsGravatar letouzey2012-07-05
* Notation: a new annotation "compat 8.x" extending "only parsing"Gravatar letouzey2012-07-05
* Bug 2767Gravatar pboutill2012-05-09
* Remove the Dp plugin.Gravatar gmelquio2012-04-17
* "A -> B" is a notation for "forall _ : A, B".Gravatar pboutill2012-04-12
* Fixing a few bugs (see #2571) related to interpretation of multiple bindersGravatar herbelin2012-04-06
* Final part of moving Program code inside the main code. Adapted add_definitio...Gravatar msozeau2012-03-14
* No more use of tauto in Init/Gravatar pboutill2012-01-19
* theories/, plugins/ and test-suite/ ported to the Arguments vernacularGravatar gareuselesinge2011-11-21
* 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