Sun, 01 Jan 2012 09:27:48 +0100 huffman merged
Fri, 30 Dec 2011 16:08:35 +0100 huffman add simp rules for bitwise word operations with 1
Sat, 31 Dec 2011 17:53:50 +0100 nipkow tuned types
Sat, 31 Dec 2011 10:15:53 +0100 krauss disabled failing sledgehammer unit test (collateral damage of 184d36538e51)
Sat, 31 Dec 2011 00:19:32 +0100 krauss disabled kodkodi in mira runs as well (cf. 493d9c4d7ed5)
Fri, 30 Dec 2011 18:14:56 +0100 berghofe merged
Fri, 30 Dec 2011 18:12:00 +0100 berghofe Made gen_dest_case more robust against eta contraction
Fri, 30 Dec 2011 17:45:13 +0100 wenzelm merged
Fri, 30 Dec 2011 11:11:57 +0100 huffman remove unnecessary intermediate lemmas
Fri, 30 Dec 2011 17:40:30 +0100 wenzelm tuned;
Fri, 30 Dec 2011 16:43:46 +0100 wenzelm eliminated old-fashioned Global_Theory.add_thms;
Fri, 30 Dec 2011 15:43:07 +0100 wenzelm simplified proof -- avoid res_inst_tac, afford plain asm_full_simp_tac;
Fri, 30 Dec 2011 14:19:58 +0100 wenzelm simplified proof;
Fri, 30 Dec 2011 13:52:07 +0100 wenzelm simplified proof;
Fri, 30 Dec 2011 12:54:55 +0100 wenzelm simplified proof;
Fri, 30 Dec 2011 12:12:16 +0100 wenzelm more parallelism;
Fri, 30 Dec 2011 12:00:10 +0100 wenzelm tuned;
Thu, 29 Dec 2011 20:32:59 +0100 wenzelm merged
Thu, 29 Dec 2011 20:31:58 +0100 wenzelm tuned -- afford slightly larger simpset in simp_defs_tac;
Thu, 29 Dec 2011 20:05:53 +0100 wenzelm tuned -- standard proofs by default;
Thu, 29 Dec 2011 19:37:24 +0100 wenzelm do not fork skipped proofs;
Thu, 29 Dec 2011 18:27:17 +0100 wenzelm clarified timeit_msg;
Thu, 29 Dec 2011 16:58:19 +0100 wenzelm tuned;
Thu, 29 Dec 2011 15:54:37 +0100 wenzelm comments;
Thu, 29 Dec 2011 18:54:07 +0100 huffman remove constant 'ccpo.lub', re-use constant 'Sup' instead
Thu, 29 Dec 2011 17:43:54 +0100 nipkow merged
Thu, 29 Dec 2011 17:43:40 +0100 nipkow tuned
Thu, 29 Dec 2011 15:14:44 +0100 haftmann conversions from sets to predicates and vice versa; extensionality on predicates
Thu, 29 Dec 2011 15:14:44 +0100 haftmann added implementation of pred_of_set
Thu, 29 Dec 2011 14:23:40 +0100 haftmann fundamental theorems on Set.bind
Thu, 29 Dec 2011 14:44:44 +0100 wenzelm updated generated files;
Thu, 29 Dec 2011 13:42:21 +0100 haftmann qualified Finite_Set.fold
Thu, 29 Dec 2011 13:41:41 +0100 haftmann qualified Finite_Set.fold
Thu, 29 Dec 2011 10:47:56 +0100 haftmann dropped redundant setup
Thu, 29 Dec 2011 10:47:56 +0100 haftmann tuned declaration
Thu, 29 Dec 2011 10:47:55 +0100 haftmann attribute code_abbrev superseedes code_unfold_post; tuned text
Thu, 29 Dec 2011 10:47:55 +0100 haftmann attribute code_abbrev superseedes code_unfold_post; tuned names and spacing
Thu, 29 Dec 2011 10:47:55 +0100 haftmann attribute code_abbrev superseedes code_unfold_post
Thu, 29 Dec 2011 10:47:55 +0100 haftmann semiring_numeral_0_eq_0, semiring_numeral_1_eq_1 now [simp], superseeding corresponding simp rules on type nat; attribute code_abbrev superseedes code_unfold_post
Thu, 29 Dec 2011 10:47:54 +0100 haftmann semiring_numeral_0_eq_0, semiring_numeral_1_eq_1 now [simp], superseeding corresponding simp rules on type nat
Wed, 28 Dec 2011 22:08:44 +0100 wenzelm merged
Wed, 28 Dec 2011 20:05:52 +0100 huffman merged
Wed, 28 Dec 2011 20:05:28 +0100 huffman restate some lemmas to respect int/bin distinction
Wed, 28 Dec 2011 19:15:28 +0100 huffman simplify some proofs
Wed, 28 Dec 2011 18:50:35 +0100 huffman add lemma word_eq_iff
Wed, 28 Dec 2011 18:33:03 +0100 huffman restate lemma word_1_no in terms of Numeral1
Wed, 28 Dec 2011 18:27:34 +0100 huffman remove recursion combinator bin_rec;
Wed, 28 Dec 2011 16:24:28 +0100 huffman simplify definition of XOR for type int;
Wed, 28 Dec 2011 16:10:49 +0100 huffman simplify definition of OR for type int;
Wed, 28 Dec 2011 16:04:58 +0100 huffman simplify definition of NOT for type int
Wed, 28 Dec 2011 13:20:46 +0100 huffman add several new tests, most of which don't work yet
Wed, 28 Dec 2011 12:55:37 +0100 huffman fix typos
Wed, 28 Dec 2011 12:52:23 +0100 huffman remove some duplicate lemmas
Wed, 28 Dec 2011 10:48:39 +0100 huffman simplify proof
Wed, 28 Dec 2011 10:30:43 +0100 huffman replace 'lemmas' with explicit 'lemma'
Wed, 28 Dec 2011 07:58:17 +0100 huffman add section headings
Tue, 27 Dec 2011 18:26:15 +0100 huffman remove duplicate lemma lists
Wed, 28 Dec 2011 20:03:13 +0100 wenzelm reverted some changes for set->predicate transition, according to "hg log -u berghofe -r Isabelle2007:Isabelle2008";
Wed, 28 Dec 2011 15:08:12 +0100 wenzelm disable kodkodi for now to prevent isatest failure of HOL-Nitpick_Examples due to 'a set constructor;
Wed, 28 Dec 2011 14:38:14 +0100 wenzelm updated platform information;
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip