aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
* Proof_type: rule now degenerates to prim_ruleGravatar letouzey2012-10-06
* Clean-up : no more Proof_type.proof_treeGravatar letouzey2012-10-06
* Clean-up of proof_type.ml : no more Nested nor abstract_tactic_boxGravatar letouzey2012-10-06
* Fix a confusion between types of locations in an untyped part of the parserGravatar letouzey2012-10-05
* Repair the configure after Hugo's last "repair" ;-)Gravatar letouzey2012-10-05
* coqtop -time : display per-command timingsGravatar letouzey2012-10-05
* More accurate timings for "Time foo"Gravatar letouzey2012-10-05
* Revert r15851 "En cours pour bug 2836".Gravatar herbelin2012-10-04
* Revert "En cours pour 'generalize in clause' et 'induction in clause'"Gravatar herbelin2012-10-04
* Repaired configure damaged in r15748 for those bash users which haveGravatar herbelin2012-10-04
* Suggest to use clean rather than archclean before recompiling.Gravatar herbelin2012-10-04
* Improving error message when abtraction over goal (abstract_list_allGravatar herbelin2012-10-04
* En cours pour 'generalize in clause' et 'induction in clause'Gravatar herbelin2012-10-04
* En cours pour bug 2836Gravatar herbelin2012-10-04
* Makefile.build: easier compilation with timings infoGravatar letouzey2012-10-04
* Getting rid of Compat in the checker.Gravatar ppedrot2012-10-04
* Adding a nominal typing layer to Metasyntax in order to clarifyGravatar ppedrot2012-10-04
* Moved Compat to parsing. This permits to break the dependency of theGravatar ppedrot2012-10-04
* Remove the unused "intel" field in Proof.proof_stateGravatar letouzey2012-10-02
* Remove some dead code in the vmGravatar letouzey2012-10-02
* Remove some more "open" and dead code thanks to OCaml4 warningsGravatar letouzey2012-10-02
* Argextend: avoid useless "open Extrawit"Gravatar letouzey2012-10-02
* avoid referring to Term in constrexpr.mli and glob_term.mliGravatar letouzey2012-10-02
* New makefile shortcuts miniopt and minibyte for coqtop + pluginsGravatar letouzey2012-10-02
* Use the library function List.substract in prev commitGravatar letouzey2012-10-02
* Added a new tactical infoH tac, that displays the names of hypothesis created...Gravatar courtieu2012-10-01
* Ltac repeat is in fact already doing progressGravatar letouzey2012-10-01
* Default hashconsing of identifiers.Gravatar ppedrot2012-09-27
* Reusing the Hashset data structure in Hashcons. Hopefully, this shouldGravatar ppedrot2012-09-26
* Incorrect commentGravatar msozeau2012-09-26
* Cleaning, renaming obscure functions and documenting in Hashcons.Gravatar ppedrot2012-09-26
* Fixing ocamldoc errorsGravatar ppedrot2012-09-25
* Added a ml-dot option to Makefile to generate dependency graph of core modulesGravatar ppedrot2012-09-25
* Fixing #2865.Gravatar ppedrot2012-09-25
* Fixing a bug introduced in Funind plugin when reorganizing the CListGravatar ppedrot2012-09-24
* Fix use of $(HASNATDYNLINK) in coq_makefile outputGravatar glondu2012-09-22
* Avoid generating ide/coqide_main*.ml as cleartext (except if READABLE_ML4 is ...Gravatar letouzey2012-09-20
* Remove broken makefile option NO_RECOMPILE_LIBGravatar letouzey2012-09-20
* Fixing Show Script issues.Gravatar ppedrot2012-09-20
* Coq_makefile fixupsGravatar pboutill2012-09-18
* More cleaning in CArray...Gravatar ppedrot2012-09-18
* More cleanup of Util: utf8 aspects moved to a new file unicode.mlGravatar letouzey2012-09-18
* Cleaning interface of Util.Gravatar ppedrot2012-09-18
* More cleaning on Utils and CList. Some parts of the code beingGravatar ppedrot2012-09-17
* MacOS integration uses lablgtkosx >= 1.1Gravatar pboutill2012-09-17
* More type-safe interface to Coq XML API.Gravatar ppedrot2012-09-17
* Move reflexivity, symmetry, and transitivity, next to f_equal, in the documen...Gravatar gmelquio2012-09-16
* Some more fixes to tactic documentation.Gravatar gmelquio2012-09-16
* Beautify tactic documentation a bit more.Gravatar gmelquio2012-09-16
* Remove superfluous spaces and commas in tactic documentation.Gravatar gmelquio2012-09-16