aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
* Fixing bug #2969 (admit failing after Grab Existential Variables dueGravatar herbelin2013-01-29
* Fixed synchronicity of filter with evar context in new_goal_with.Gravatar herbelin2013-01-29
* Renaming evar_env/evar_unfiltered_env into evar_filtered_env/evar_envGravatar herbelin2013-01-29
* Fixed bug #2966 (de Bruijn error in computation of heads for coercions).Gravatar herbelin2013-01-28
* Actually adding backtrace handling.Gravatar ppedrot2013-01-28
* Added backtrace primitives.Gravatar ppedrot2013-01-28
* Uniformization of the "anomaly" command.Gravatar ppedrot2013-01-28
* Fixing one part of #2830 (anomaly "defined twice" due to nested calls toGravatar herbelin2013-01-28
* native_compute: Fixed dependencies compilation order.Gravatar mdenes2013-01-28
* Added backtrace information to anomaliesGravatar ppedrot2013-01-28
* Ordered evars by level of dependency in the merging phase of unificationGravatar herbelin2013-01-27
* Improving formatting of output of "Test table".Gravatar herbelin2013-01-27
* Fixed bug #2967 (some missing check on ill-formed recursive notation strings).Gravatar herbelin2013-01-27
* Slightly improving some debugging printing and error message for modules.Gravatar herbelin2013-01-27
* Avoid failure in debugger when printing Ltac names.Gravatar herbelin2013-01-27
* updating ide/coq documentationGravatar ppedrot2013-01-26
* Monadification of coqtop queries in CoqIDEGravatar ppedrot2013-01-26
* Uniformization of Coq tasksGravatar ppedrot2013-01-26
* Better handling of escape find in CoqIDEGravatar ppedrot2013-01-25
* Better Undo/Redo mechanismGravatar ppedrot2013-01-25
* Trying to fix CoqIDE undo/redo mechanismGravatar ppedrot2013-01-25
* Fixing autocompletion in CoqIDEGravatar ppedrot2013-01-25
* Fixup last commitGravatar ppedrot2013-01-25
* Hugo request: CoqIDE find on enterGravatar ppedrot2013-01-25
* Reductionops: whd_state_gen can take and answers a cst_stack tooGravatar pboutill2013-01-24
* Fixed parsing of -no-native-compiler flag.Gravatar mdenes2013-01-24
* Native compiler: warnings were not turned off for OCaml 3.11Gravatar mdenes2013-01-24
* Coqide: limit read buffer size to 4096 (pipe size in win32)Gravatar letouzey2013-01-23
* Coqide: avoid potentially blocking read on coqtop channelGravatar letouzey2013-01-22
* Added .native to .gitignoreGravatar ppedrot2013-01-22
* New implementation of the conversion test, using normalization by evaluation toGravatar mdenes2013-01-22
* Revert "remove -rectypes except for term.ml"Gravatar mdenes2013-01-22
* - Fix evarconv so that we have complete eta-conversion:Gravatar msozeau2013-01-22
* Fix bug 2958: Inductive deep in in clause are impossibleGravatar pboutill2013-01-21
* Last test-suite not in Symmetric Patterns syntaxGravatar pboutill2013-01-21
* I forget to use git log before git svn dcommit ...Gravatar pboutill2013-01-18
* Evarconv: Check stack before term in Canonical Structure approuvalGravatar pboutill2013-01-18
* Unset Asymmetric PatternsGravatar pboutill2013-01-18
* Revert "coq_makefile: use coqdep instead of ocamldep on .ml4 files"Gravatar pboutill2013-01-18
* Envar: in w32, add .exe when searching for caml binariesGravatar letouzey2013-01-12
* Coqmktop and camlp4 : sequel to commit 16113Gravatar letouzey2013-01-12
* Coq_makefile: quoting pathsGravatar pboutill2013-01-07
* Coq_makefile: -extra & -phony-extra for user defined makefile ruleGravatar pboutill2013-01-07
* Fixup notation printing in patternsGravatar pboutill2013-01-07
* * Kernel/Terms:Gravatar regisgia2013-01-06
* Avoiding collision between Camlp4 Loc.Exc_located and Coq's Loc.Exc_located.Gravatar herbelin2012-12-22
* nat_iter n f x -> nat_rect _ x (fun _ => f) nGravatar pboutill2012-12-21
* Yet a new reduction tactic in Coq : cbnGravatar pboutill2012-12-21
* Awful heuristic to refold mutual fixpoint in reductionopsGravatar pboutill2012-12-21
* Fixup and comment reductionopsGravatar pboutill2012-12-21