Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
tuned proofs;
2012-02-21, by wenzelm
more robust visible_range: allow empty view;
2012-02-21, by wenzelm
misc tuning;
2012-02-21, by wenzelm
merged;
2012-02-21, by wenzelm
made SML/NJ happy;
2012-02-21, by wenzelm
tuned proofs;
2012-02-21, by wenzelm
merged
2012-02-21, by wenzelm
tuned proofs;
2012-02-21, by wenzelm
approximate Perspective.full within the bounds of the JVM;
2012-02-21, by wenzelm
misc tuning;
2012-02-21, by wenzelm
invoke later to reduce chance of causing deadlock;
2012-02-21, by wenzelm
misc tuning;
2012-02-21, by wenzelm
separate module for text status overview;
2012-02-21, by wenzelm
overview.delay_repaint: avoid wasting GUI cycles via update_delay;
2012-02-21, by wenzelm
tuned;
2012-02-21, by wenzelm
merged
2012-02-21, by berghofe
merged
2012-02-21, by berghofe
Fixed bugs:
2012-02-20, by berghofe
merged
2012-02-21, by bulwahn
subtype preprocessing in Quickcheck;
2012-02-21, by bulwahn
adding parsing of an optional predicate with quickcheck_generator command
2012-02-21, by bulwahn
updated generated files (cf. 8d51b375e926);
2012-02-21, by wenzelm
merged;
2012-02-21, by wenzelm
add missing lemmas to compute_div_mod
2012-02-21, by huffman
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
2012-02-21, by huffman
avoid using constant Int.neg
2012-02-21, by huffman
renamed ex/Numeral.thy to ex/Numeral_Representation.thy
2012-02-21, by huffman
reverting changesets from 5d33a3269029 on: change of order of declaration of classical rules makes serious problems
2012-02-21, by haftmann
tuned whitespace
2012-02-20, by haftmann
tuned proof
2012-02-20, by haftmann
tuned proof
2012-02-19, by haftmann
distributed lattice properties of predicates to places of instantiation
2012-02-19, by haftmann
removing some unnecessary premises from Divides
2012-02-20, by bulwahn
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
2012-02-20, by huffman
observe HEIGHT of overview ticks;
2012-02-20, by wenzelm
more careful painting of overview component: more precise and more efficient;
2012-02-20, by wenzelm
clarified initial process startup errors: recover image load failure message (cf. 2cb7e34f6096) and suppress accidental output from raw ML toplevel;
2012-02-20, by wenzelm
use qualified constant names instead of suffixes (from Florian Haftmann)
2012-02-20, by huffman
tuned proofs
2012-02-18, by haftmann
tuned
2012-02-12, by haftmann
brute-force adjustion
2012-02-11, by haftmann
tuned whitespace
2012-02-11, by haftmann
tuned
2012-02-11, by haftmann
tuned
2012-02-10, by haftmann
tuned code
2012-02-10, by haftmann
dropped whitespace
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
corrected typo
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
notepad is more appropriate here
2012-02-12, by haftmann
corrected treatment of applications of built-in functions to higher-order terms
2012-02-18, by boehmes
NEWS
2012-02-18, by krauss
merged
2012-02-18, by krauss
added congruence rules for Option.{map|bind}
2012-02-18, by krauss
updated generated documents
2012-02-18, by haftmann
avoid redefinition of @{theory} antiquotation
2012-02-18, by haftmann
update of generated documents
2012-02-18, by haftmann
tuned whitespace
2012-02-18, by haftmann
clarified
2012-02-18, by haftmann
corrected spelling
2012-02-18, by haftmann
clarified
2012-02-18, by haftmann
more precise semantics of "theory" antiquotation
2012-02-18, by haftmann
tuned import
2012-02-18, by haftmann
dropped references to obsolete theories
2012-02-18, by haftmann
adjusted to set type constructor
2012-02-18, by haftmann
tuned whitespace
2012-02-18, by haftmann
more explicit error on malformed abstract equation; dropped dead code; tuned signature
2012-02-18, by haftmann
simplified configuration options for syntax ambiguity;
2012-02-17, by wenzelm
retain default of Syntax.ambiguity, according to 2bd54d4b5f3d (despite earlier versions);
2012-02-17, by wenzelm
more antiquotations;
2012-02-16, by wenzelm
more symbols;
2012-02-16, by wenzelm
tuned imports;
2012-02-16, by wenzelm
tuned proofs;
2012-02-16, by wenzelm
simplified configuration options for syntax ambiguity;
2012-02-16, by wenzelm
merged
2012-02-16, by wenzelm
removing unnecessary premise from diff_single_insert
2012-02-16, by bulwahn
explicit is better than implicit;
2012-02-16, by wenzelm
more uniform / portable representation of the idea of "copy_dir" (NB: cp -f dereferences symlinks on GNU/Linux, but does not on old-school Unixen including BSD/Mac OS X);
2012-02-16, by wenzelm
simplifying proof
2012-02-16, by bulwahn
removing unnecessary premises in theorems of List theory
2012-02-16, by bulwahn
tuning mutabelle script
2012-02-16, by bulwahn
adding documentation for abort_potential option in quickcheck
2012-02-16, by bulwahn
renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in conformance with similar operations in structure Term and Logic;
2012-02-15, by wenzelm
discontinued Drule.term_rule, which tends to cause confusion due to builtin cterm_of (NB: the standard morphisms already provide a separate term component);
2012-02-15, by wenzelm
uniform Isar source formatting for this file;
2012-02-15, by wenzelm
clarified outer syntax "constdecl", which is only local to some rail diagrams;
2012-02-15, by wenzelm
discontinued obsolete "prems" fact;
2012-02-15, by wenzelm
eliminated slightly odd / obsolete DETERM_UNTIL, DETERM_UNTIL_SOLVED (cf. 941afb897532, ea0668a1c0ba);
2012-02-15, by wenzelm
removed obsolete files;
2012-02-15, by wenzelm
more basic simplification, eliminated slightly odd tactic style from 1995 (cf. ea0668a1c0ba);
2012-02-15, by wenzelm
removed dead code;
2012-02-15, by wenzelm
updated listrel (cf. 80dccedd6c14);
2012-02-15, by wenzelm
removed redundant cut_inst_tac -- already covered in implementation manual;
2012-02-15, by wenzelm
updated rewrite_goals_rule, rewrite_rule;
2012-02-15, by wenzelm
NEWS;
2012-02-15, by wenzelm
updated refs;
2012-02-15, by wenzelm
renamed "xstr" to "str_token";
2012-02-15, by wenzelm
merged
2012-02-14, by wenzelm
don't report spurious LEO-II errors
2012-02-14, by blanchet
better error message
2012-02-14, by blanchet
removing debug code in mutabelle
2012-02-14, by bulwahn
adding abort_potential functionality in quickcheck
2012-02-14, by bulwahn
adding abort_potential configuration in Quickcheck
2012-02-14, by bulwahn
clarified bires_inst_tac: retain internal exceptions;
2012-02-14, by wenzelm
tuned signature;
2012-02-14, by wenzelm
more conventional tactic setup -- avoid low-level Thm.dest_state and spurious warnings about it;
2012-02-14, by wenzelm
more conventional tactic setup;
2012-02-14, by wenzelm
eliminated odd/obsolete innermost_params (cf. a77ad6c86564, 3458b0e955ac);
2012-02-14, by wenzelm
prefer high-level elim_format;
2012-02-14, by wenzelm
discontinued unused MRL -- in correspondence with section "2.4.2 Rule composition" in the implementation manual;
2012-02-14, by wenzelm
method setup;
2012-02-14, by wenzelm
simplified use of tacticals;
2012-02-14, by wenzelm
comment;
2012-02-14, by wenzelm
tuned signature, according to actual usage of these operations;
2012-02-14, by wenzelm
tuned signature;
2012-02-14, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip