| Commit message (Expand) | Author | Age |
* | Move setoid_rewrite to its own module and do some clean up in | msozeau | 2009-04-07 |
* | Fix behavior on newlines with parse-comments and also do [] escaping as | msozeau | 2009-04-06 |
* | correction bug 2085 | soubiran | 2009-04-06 |
* | Display the content of the list instead of "<list>" when an idtac | herbelin | 2009-04-05 |
* | Fix obvious bug in evars_of_named_context. | msozeau | 2009-04-03 |
* | Ocamlbuild: option for (not) building coqide, better log messages | letouzey | 2009-04-03 |
* | Makefile: ocamlbuild's _build is not traversed by find, and removed by make c... | letouzey | 2009-04-03 |
* | Ocamlbuild: improvements suggested by N. Pouillard | letouzey | 2009-04-03 |
* | Fix auto so that Extern tactics associated to no patterns can apply to | msozeau | 2009-03-31 |
* | Committed patch sent by Samuel Bronson on Mar 14 2009 to take care of | herbelin | 2009-03-31 |
* | Complementary fix to have ocamlopt_shared_os5fix.sh working correctly | herbelin | 2009-03-31 |
* | Fix the fix script for ocamlopt -shared in MacOS 10.5 (remarks by Hugo) | letouzey | 2009-03-30 |
* | Update CHANGES | glondu | 2009-03-30 |
* | Document new quote construction | glondu | 2009-03-30 |
* | Add tests for quote | glondu | 2009-03-30 |
* | Add a more general quote construction | glondu | 2009-03-30 |
* | Fix some typos and spaces | glondu | 2009-03-30 |
* | Csdpcert: adaptation after last commit | letouzey | 2009-03-29 |
* | Micromega: improvement of the code obtained by extraction | letouzey | 2009-03-29 |
* | ocamlbuild: many improvements (macos 10.5 fix, correct dllpath, etc) | letouzey | 2009-03-29 |
* | Avoid inadvertent declaration of "on" as a keyword. New syntax is | msozeau | 2009-03-29 |
* | Fix useless redeclaration of a tactic name when UpdateTac is replayed. | msozeau | 2009-03-28 |
* | Rewrite of Program Fixpoint to overcome the previous limitations: | msozeau | 2009-03-28 |
* | Fix bug #2056 (discharge bug). | msozeau | 2009-03-28 |
* | Fix static compilation of numeral syntax (typo in _mod files, sorry ...) | letouzey | 2009-03-28 |
* | ZArith/Int: no need to load romega here (but rather in FullAVL) | letouzey | 2009-03-28 |
* | ZMicromega: useless dependency toward ZArith.Int | letouzey | 2009-03-28 |
* | Coqdep: some dead code and code move (first experiment with Oug) | letouzey | 2009-03-27 |
* | Parsing files for numerals (+ ascii/string) moved into plugins | letouzey | 2009-03-27 |
* | Remove unused mli files | letouzey | 2009-03-27 |
* | GroebnerZ: no more admitted lemmas | letouzey | 2009-03-27 |
* | Ocamlbuild: 1st reasonably complete version (rules for binaries + plugins + vo) | letouzey | 2009-03-26 |
* | Fixes in Program well-founded definitions: | msozeau | 2009-03-26 |
* | ocamlbuild: coqide, coqchk, a bit of .vo | letouzey | 2009-03-26 |
* | Coqdep_boot: one line with bad indentation | letouzey | 2009-03-26 |
* | Protect typeset arguments in titles in LaTeX output (fixes compilation | msozeau | 2009-03-26 |
* | clean revision and coqdep_boot, too | lmamane | 2009-03-26 |
* | bin/coq-{parser,interface}: use this coqtop, not the first in $PATH | lmamane | 2009-03-26 |
* | make coqdep_boot in stage1, not stage2 | lmamane | 2009-03-25 |
* | Fix coqdoc bugs reported by Ian Lynagh. | msozeau | 2009-03-24 |
* | ocamlbuild improvements + minor makefile fix | letouzey | 2009-03-24 |
* | pretty.mll of coqdoc becomes cpretty.mll (avoid clash with a camlp5 file) | letouzey | 2009-03-24 |
* | - Fixed bug 2058 (as much as possible - the syntax of "pose (f binders := ...)" | herbelin | 2009-03-23 |
* | Backport from v8.2 branch of 11986 (interpretation of quantified | herbelin | 2009-03-22 |
* | Compromise wrt introduction-names compatibility issue after addition | herbelin | 2009-03-22 |
* | More elaborate handling of newlines in Gallina mode. Support inline | msozeau | 2009-03-22 |
* | coqdoc fixes and support for parsing regular comments (request by | msozeau | 2009-03-22 |
* | Many changes in the Makefile infrastructure + a beginning of ocamlbuild | letouzey | 2009-03-20 |
* | Makefile: avoid $(ML4FILES:.ml4=.ml) since this is $(ML4FILESML) | letouzey | 2009-03-20 |
* | replaced dir_load by load_file because dir_load does not raise an exception w... | barras | 2009-03-20 |