aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
* Locating errors from consider_remaining_unif_problems if possibleGravatar herbelin2013-02-17
* Added propagation of evars unification failure reasons for betterGravatar herbelin2013-02-17
* Revised the Ltac trace mechanism so that trace breaking due toGravatar herbelin2013-02-17
* Fix extraction of inductive types that Coq auto-detects to be in PropGravatar letouzey2013-02-14
* CoqIDE: Adding escape reaction to replace widgetGravatar ppedrot2013-02-13
* Fixing autocompletion lock in CoqIDEGravatar ppedrot2013-02-13
* make validate repaired via a temporary fix for #2949Gravatar letouzey2013-02-13
* Checker: re-sync vo structures after Maxime's commit 16136Gravatar letouzey2013-02-12
* Fixing bug in native compiler with let patterns in fixpoint definitions.Gravatar mdenes2013-02-11
* Useless use of hooks in VernacDefinition. In addition, this wasGravatar ppedrot2013-02-10
* Splitted Evarutil in two filesGravatar ppedrot2013-02-10
* Moved code from Pretype_error to EvarutilGravatar ppedrot2013-02-10
* Revert "Ordered evars by level of dependency in the merging phase of unificat...Gravatar herbelin2013-02-05
* Fixed bug #2981 (anomaly NotASort in Retyping due to collision betweenGravatar herbelin2013-02-05
* Fixing coqchk compilation after commit r16183Gravatar ppedrot2013-02-03
* v8.4: Granting bug/wish #2976 (turning anomaly on input_value into nice message)Gravatar herbelin2013-02-01
* Fixed #2970 (made that remember's eqn name is interpretable as an ltac var).Gravatar herbelin2013-01-29
* Added a file for testing regression of bug #2955 (anomaly in simpl inGravatar herbelin2013-01-29
* No reason a priori for using unfiltered env for printingGravatar herbelin2013-01-29
* 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