Wed, 12 May 2010 23:53:56 +0200 boehmes deleted SMT translation files (to be replaced by a simplified version)
Wed, 12 May 2010 23:53:55 +0200 boehmes move the addition of extra facts into a separate module
Wed, 12 May 2010 23:53:54 +0200 boehmes normalize numerals: also rewrite Numeral0 into 0
Wed, 12 May 2010 23:53:53 +0200 boehmes added missing rewrite rules for natural min and max
Wed, 12 May 2010 23:53:52 +0200 boehmes rewrite bool case expressions as if expression
Wed, 12 May 2010 23:53:51 +0200 boehmes simplified normalize_rule and moved it further down in the code
Wed, 12 May 2010 23:53:50 +0200 boehmes merged addition of rules into one function
Wed, 12 May 2010 23:53:49 +0200 boehmes added simplification for distinctness of small lists
Wed, 12 May 2010 23:53:48 +0200 boehmes moved the addition of DLO tactic into the Z3 theory (DLO is required only for Z3 proof reconstruction)
Fri, 14 May 2010 19:53:36 +0200 wenzelm added Proofterm.unconstrain_thm_proof for Thm.unconstrainT -- loosely based on the version by krauss/schropp;
Thu, 13 May 2010 21:36:38 +0200 wenzelm conditionally unconstrain thm proofs -- loosely based on the version by krauss/schropp;
Thu, 13 May 2010 21:17:09 +0200 wenzelm the_classrel/the_arity: avoid Thm.transfer for proofterm version -- theory might already have become stale within the proof_body future;
Thu, 13 May 2010 20:15:59 +0200 wenzelm avoid redundant rebinding of name/prop -- probably introduced accidentally in 80bb72a0f577;
Thu, 13 May 2010 18:47:07 +0200 wenzelm raise Fail uniformly for proofterm errors, which appear to be rather low-level;
Thu, 13 May 2010 18:22:10 +0200 wenzelm unconstrainT operations on proofs, according to krauss/schropp;
Thu, 13 May 2010 17:25:53 +0200 wenzelm added Proofterm.get_name variants according to krauss/schropp;
Wed, 12 May 2010 22:43:05 +0200 wenzelm conditional structure SingleAssignment;
Wed, 12 May 2010 17:10:53 +0200 wenzelm merged
Wed, 12 May 2010 15:31:43 +0200 haftmann merged
Wed, 12 May 2010 15:27:15 +0200 haftmann tuned proofs and fact and class names
Wed, 12 May 2010 13:51:22 +0200 haftmann tuned fact collection names and some proofs
Wed, 12 May 2010 12:31:52 +0200 haftmann grouped local statements
Wed, 12 May 2010 12:31:51 +0200 haftmann tuned test problems
Wed, 12 May 2010 16:45:59 +0200 wenzelm merged
Wed, 12 May 2010 15:25:23 +0200 nipkow merged
Wed, 12 May 2010 15:25:02 +0200 nipkow simplified proof
Wed, 12 May 2010 16:44:49 +0200 wenzelm modernized specifications;
Wed, 12 May 2010 15:25:58 +0200 wenzelm updated/unified some legacy warnings;
Wed, 12 May 2010 15:23:38 +0200 wenzelm tuned;
Wed, 12 May 2010 14:52:23 +0200 wenzelm do not emit legacy_feature warnings here -- users have no chance to disable them;
Wed, 12 May 2010 14:17:26 +0200 wenzelm removed obsolete CVS Ids;
Wed, 12 May 2010 14:02:50 +0200 wenzelm removed some obsolete admin stuff;
Wed, 12 May 2010 14:02:19 +0200 wenzelm check NEWS;
Wed, 12 May 2010 13:54:49 +0200 wenzelm removed obsolete CVS Ids;
Wed, 12 May 2010 13:52:34 +0200 wenzelm updated some version numbers;
Wed, 12 May 2010 13:34:24 +0200 wenzelm minor tuning;
Wed, 12 May 2010 13:21:23 +0200 wenzelm reverted parts of 7902dc7ea11d -- note that NEWS of published Isabelle releases are essentially read-only;
Wed, 12 May 2010 12:51:32 +0200 wenzelm merged
Wed, 12 May 2010 12:20:16 +0200 haftmann merged
Wed, 12 May 2010 12:09:28 +0200 haftmann modernized specifications; tuned reification
Wed, 12 May 2010 11:18:42 +0200 haftmann merged
Wed, 12 May 2010 11:17:59 +0200 haftmann added lemmas concerning last, butlast, insort
Wed, 12 May 2010 11:30:18 +0200 Cezary Kaliszyk Remove RANGE_WARN
Wed, 12 May 2010 11:13:33 +0200 hoelzl clarified NEWS entry
Wed, 12 May 2010 11:08:15 +0200 hoelzl merged
Wed, 12 May 2010 11:07:46 +0200 hoelzl added NEWS entry
Tue, 11 May 2010 19:19:45 +0200 hoelzl Added atLeastAtMost_singleton_iff, atLeastAtMost_singleton'
Tue, 11 May 2010 19:21:39 +0200 hoelzl Add rules directly to the corresponding class locales instead.
Tue, 11 May 2010 19:21:05 +0200 hoelzl Removed usage of normalizating locales.
Tue, 11 May 2010 21:55:41 -0700 huffman speed up some proofs, fixing linarith_split_limit warnings
Tue, 11 May 2010 19:38:16 -0700 huffman fix some linarith_split_limit warnings
Tue, 11 May 2010 19:01:35 -0700 huffman include iszero_simps in semiring_norm just once (they are already included in rel_simps)
Tue, 11 May 2010 19:00:32 -0700 huffman fix duplicate simp rule warning
Tue, 11 May 2010 18:06:58 -0700 huffman no more RealPow.thy (remaining lemmas moved to RealDef.thy)
Tue, 11 May 2010 17:20:11 -0700 huffman merged
Tue, 11 May 2010 12:38:07 -0700 huffman simplify code for emptiness check
Tue, 11 May 2010 12:05:19 -0700 huffman removed lemma real_sq_order; use power2_le_imp_le instead
Tue, 11 May 2010 21:27:09 +0200 haftmann merged
Tue, 11 May 2010 19:06:18 +0200 haftmann merged
Tue, 11 May 2010 19:00:16 +0200 haftmann represent de-Bruin indices simply by position in list
Tue, 11 May 2010 18:46:03 +0200 haftmann tuned reification functions
Tue, 11 May 2010 18:31:36 +0200 haftmann tuned code; toward a tightended interface with generated code
Tue, 11 May 2010 11:58:34 -0700 huffman fix spelling of 'superseded'
Tue, 11 May 2010 11:57:14 -0700 huffman NEWS: removed theory PReal
Tue, 11 May 2010 11:40:39 -0700 huffman collected NEWS updates for HOLCF
Tue, 11 May 2010 11:02:56 -0700 huffman merged
Tue, 11 May 2010 09:10:31 -0700 huffman move floor lemmas from RealPow.thy to RComplete.thy
Tue, 11 May 2010 07:58:48 -0700 huffman add lemma tendsto_Complex
Tue, 11 May 2010 06:30:48 -0700 huffman move some theorems from RealPow.thy to Transcendental.thy
Tue, 11 May 2010 06:27:06 -0700 huffman add lemma power2_eq_1_iff; generalize some other lemmas
Mon, 10 May 2010 21:33:48 -0700 huffman minimize imports
Mon, 10 May 2010 21:27:52 -0700 huffman move lemma real_mult_is_one to Rings.thy, renamed to square_eq_1_iff
Wed, 12 May 2010 12:50:00 +0200 wenzelm clarified Pretty.font_metrics;
Wed, 12 May 2010 11:31:05 +0200 wenzelm format as topmost list of "divs", not just adjacent "spans" -- for proper line breaking;
Wed, 12 May 2010 11:28:52 +0200 wenzelm tuned;
Tue, 11 May 2010 23:36:06 +0200 wenzelm more precise pretty printing based on actual font metrics;
Tue, 11 May 2010 23:09:49 +0200 wenzelm predefined spaces;
Tue, 11 May 2010 17:55:19 +0200 wenzelm merged
Tue, 11 May 2010 15:47:31 +0200 wenzelm support Isabelle plugin properties with defaults;
Tue, 11 May 2010 08:52:22 +0100 Christian Urban merged
Tue, 11 May 2010 07:45:47 +0100 Christian Urban tuned proof so that no simplifier warning is printed
Tue, 11 May 2010 08:36:02 +0200 haftmann renamed former Int.int_induct to Int.int_of_nat_induct, former Presburger.int_induct to Int.int_induct: is more conservative and more natural than the intermediate solution
Tue, 11 May 2010 08:30:02 +0200 haftmann merged
Tue, 11 May 2010 08:29:42 +0200 haftmann tuned
Tue, 11 May 2010 08:29:42 +0200 haftmann theorem Presburger.int_induct has been renamed to Int.int_bidirectional_induct
Mon, 10 May 2010 15:33:32 +0200 haftmann tuned; dropped strange myassoc2
Mon, 10 May 2010 15:24:43 +0200 haftmann stylized COOPER exception
Mon, 10 May 2010 15:21:13 +0200 haftmann simplified oracle
Mon, 10 May 2010 15:00:53 +0200 haftmann shorten names
Mon, 10 May 2010 14:57:04 +0200 haftmann updated references to ML files
Mon, 10 May 2010 14:55:06 +0200 haftmann only one module fpr presburger method
Mon, 10 May 2010 14:55:04 +0200 haftmann moved int induction lemma to theory Int as int_bidirectional_induct
Mon, 10 May 2010 14:18:41 +0200 haftmann tuned theory text; dropped unused lemma
Mon, 10 May 2010 14:11:50 +0200 haftmann one structure is better than three
Mon, 10 May 2010 13:58:18 +0200 haftmann less complex organization of cooper source code
Mon, 10 May 2010 12:25:49 +0200 haftmann dropped unused bindings; avoid open (documents dependency on generated code more explicitly)
Mon, 10 May 2010 14:53:33 -0700 huffman add real_mult_commute to legacy theorem names
Mon, 10 May 2010 12:12:58 -0700 huffman new construction of real numbers using Cauchy sequences
Mon, 10 May 2010 11:47:56 -0700 huffman add more credits to ex/Dedekind_Real.thy
Mon, 10 May 2010 11:30:05 -0700 huffman put construction of reals using Dedekind cuts in HOL/ex
Tue, 11 May 2010 10:36:50 +0200 wenzelm disable two stage save by default, to avoid change of file permissions (notably the dreaded executable bit on Cygwin);
Mon, 10 May 2010 23:46:49 +0200 wenzelm simple dialogs: ensure Swing thread;
Mon, 10 May 2010 23:36:47 +0200 wenzelm font size re-adjustment according to Lobo internals;
Mon, 10 May 2010 22:29:27 +0200 wenzelm Scala for Netbeans 6.8v1.1.0rc2;
Mon, 10 May 2010 22:27:58 +0200 wenzelm more convenient get_font;
Mon, 10 May 2010 20:53:06 +0200 wenzelm renamed Config.get_thy to Config.get_global etc. to indicate that this is not the real thing;
Mon, 10 May 2010 17:37:32 +0200 wenzelm more convenient look-and-feel setup;
Mon, 10 May 2010 17:29:19 +0200 wenzelm more convenient get_font;
Mon, 10 May 2010 17:07:47 +0200 wenzelm explicit getLines(n) ensures platform-independence -- our files follow the POSIX standard, not DOS;
Mon, 10 May 2010 15:18:57 +0200 wenzelm updated to jedit 4.3.2;
Mon, 10 May 2010 15:01:25 +0200 wenzelm ignore spurious TIMEOUT messages, maybe caused by change of actor semantics in scala-2.8;
Mon, 10 May 2010 15:00:11 +0200 wenzelm adapted to scala-2.8.0.RC2;
Mon, 10 May 2010 09:54:41 +0200 wenzelm merged
Sun, 09 May 2010 23:57:56 -0700 huffman real_mult_commute -> mult_commute
Sun, 09 May 2010 22:51:11 -0700 huffman avoid using real-specific versions of generic lemmas
Sun, 09 May 2010 17:47:43 -0700 huffman avoid using real-specific versions of generic lemmas
Sun, 09 May 2010 14:21:44 -0700 huffman remove a couple of redundant lemmas; simplify some proofs
Sun, 09 May 2010 09:39:01 -0700 huffman merged
Sat, 08 May 2010 17:06:58 -0700 huffman add lemmas one_less_inverse and one_le_inverse
Sun, 09 May 2010 15:28:44 +0200 krauss do not redeclare [simp] rules, to avoid "duplicate rewrite rule" warnings
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip