Wed, 11 Jan 2012 18:02:59 +0100 wenzelm updated generated file -- change of printed case syntax probably due to f805747f8571;
Wed, 11 Jan 2012 17:30:34 +0100 wenzelm actually try to preserve names given by user (cf. 463b594e186a);
Wed, 11 Jan 2012 16:47:30 +0100 wenzelm updated example -- List.foldl is no longer defined via primrec;
Wed, 11 Jan 2012 16:25:34 +0100 wenzelm more qualified names;
Wed, 11 Jan 2012 16:23:59 +0100 wenzelm refer to imp_cong from HOL, not Drule (!) -- cf. 4ed94d92ae19;
Wed, 11 Jan 2012 15:12:57 +0100 wenzelm more robust ISABELLE_HOME_USER for repository versions -- some versions of Emacs interpret foo//bar as /bar even on the command-line (unlike regular POSIX semantics);
Wed, 11 Jan 2012 00:05:31 +0100 berghofe merged
Wed, 11 Jan 2012 00:01:54 +0100 berghofe Removed strange hack introduced in b27e93132603, since equivariance
Tue, 10 Jan 2012 23:59:37 +0100 berghofe Replaced perm_set_eq by perm_set_def
Tue, 10 Jan 2012 23:58:10 +0100 berghofe Corrected pt_set_inst, added missing cp_set_inst, deleted obsolete
Tue, 10 Jan 2012 23:49:53 +0100 berghofe Reverted several lemmas involving sets to the state before the
Tue, 10 Jan 2012 23:26:27 +0100 wenzelm clarified Isabelle_Rendering vs. physical painting;
Tue, 10 Jan 2012 18:12:55 +0100 berghofe pred_subset_eq and SUP_UN_eq2 are now standard pred_set_conv rules
Tue, 10 Jan 2012 18:12:03 +0100 berghofe pred_subset/equals_eq are now standard pred_set_conv rules
Tue, 10 Jan 2012 18:09:09 +0100 berghofe Declared pred_equals/subset_eq, sup_Un_eq and SUP_UN_eq(2) as pred_set_conv rules
Tue, 10 Jan 2012 17:14:25 +0100 huffman merged
Tue, 10 Jan 2012 15:43:16 +0100 huffman add simp rules for set_bit and msb applied to 0 and 1
Tue, 10 Jan 2012 14:48:42 +0100 huffman add simp rule test_bit_1
Tue, 10 Jan 2012 15:48:10 +0100 bulwahn proper hiding of facts and constants in AList_Impl and AList theory
Tue, 10 Jan 2012 10:48:39 +0100 bulwahn NEWS
Tue, 10 Jan 2012 10:18:08 +0100 bulwahn adding quickcheck examples with multisets
Tue, 10 Jan 2012 10:17:09 +0100 bulwahn improving code generation for multisets; adding exhaustive quickcheck generators for multisets
Tue, 10 Jan 2012 10:17:07 +0100 bulwahn adding theory association lists with invariant
Mon, 09 Jan 2012 23:11:28 +0100 wenzelm command status color via regular markup;
Mon, 09 Jan 2012 23:09:03 +0100 wenzelm proper cumulation of bulk arguments;
Mon, 09 Jan 2012 23:08:33 +0100 wenzelm tuned;
Mon, 09 Jan 2012 18:33:55 +0100 blanchet merge
Mon, 09 Jan 2012 18:32:56 +0100 blanchet revert unintended "sledgehammer" call
Mon, 09 Jan 2012 18:29:42 +0100 wenzelm prefer antiquotations;
Mon, 09 Jan 2012 14:47:18 +0100 wenzelm misc tuning and reformatting;
Mon, 09 Jan 2012 14:26:13 +0100 wenzelm updated generated file;
Mon, 09 Jan 2012 13:48:14 +0100 nipkow Added termination to IMP Abs_Int
Mon, 09 Jan 2012 11:41:38 +0100 nipkow added lemmas
Sat, 07 Jan 2012 20:44:23 +0100 haftmann massaging of code setup for sets
Sat, 07 Jan 2012 20:18:56 +0100 haftmann dropped theory More_Set
Sat, 07 Jan 2012 20:18:56 +0100 haftmann use Inf/Sup_bool_def/apply as code equations
Sat, 07 Jan 2012 21:19:53 +0100 nipkow tuned
Sat, 07 Jan 2012 12:39:46 +0100 wenzelm accumulate status as regular markup for command range;
Sat, 07 Jan 2012 11:45:53 +0100 haftmann corrected slip
Sat, 07 Jan 2012 09:32:18 +0100 haftmann tuned
Sat, 07 Jan 2012 09:32:01 +0100 haftmann restore convenient code_abbrev declarations (particulary important if List.set is not the formal constructor for sets)
Fri, 06 Jan 2012 22:16:25 +0100 haftmann moved lemmas about List.set and set operations to List theory
Fri, 06 Jan 2012 22:16:01 +0100 haftmann moved lemmas about List.set and set operations to List theory
Fri, 06 Jan 2012 21:48:45 +0100 haftmann incorporated various theorems from theory More_Set into corpus
Fri, 06 Jan 2012 21:48:45 +0100 haftmann consolidated various theorem names relating to Finite_Set.fold and List.fold combinators
Fri, 06 Jan 2012 20:48:52 +0100 wenzelm merged
Fri, 06 Jan 2012 20:39:50 +0100 haftmann farewell to theory More_List
Fri, 06 Jan 2012 11:15:02 +0100 haftmann dropped unused nth_map
Fri, 06 Jan 2012 10:53:52 +0100 haftmann more explicit NEWS
Fri, 06 Jan 2012 20:18:49 +0100 wenzelm refined case syntax again, improved treatment of constructors without arguments, e.g. "case a of (True, x) => x";
Fri, 06 Jan 2012 19:24:23 +0100 wenzelm tuned;
Fri, 06 Jan 2012 17:44:42 +0100 wenzelm improved list comprehension syntax: more careful treatment of position constraints, which enables PIDE markup;
Fri, 06 Jan 2012 16:45:19 +0100 wenzelm tuned -- more direct @{type_name set} (NB: binder_tr' retains the original non-syntax type for the bound/free variable);
Fri, 06 Jan 2012 16:42:15 +0100 wenzelm recovered case syntax for of_int, also with source positions (appears to be unused nonetheless);
Fri, 06 Jan 2012 15:19:17 +0100 wenzelm more careful treatment of outermost constraints, e.g. constructors without arguments (despite loss of positions for catch-all variables);
Fri, 06 Jan 2012 11:27:49 +0100 wenzelm proper refs;
Fri, 06 Jan 2012 10:19:49 +0100 haftmann incorporated canonical fold combinator on lists into body of List theory; refactored passages on List.fold(l/r)
Fri, 06 Jan 2012 10:19:49 +0100 haftmann incorporated canonical fold combinator on lists into body of List theory; refactored passages on List.fold(l/r); tuned quotes
Fri, 06 Jan 2012 10:19:48 +0100 haftmann prefer listsum over foldl plus 0
Fri, 06 Jan 2012 10:19:48 +0100 haftmann prefer concat over foldl append []
Fri, 06 Jan 2012 10:19:47 +0100 haftmann tuned proofs
Sun, 01 Jan 2012 15:44:15 +0100 haftmann interaction of set operations for execution and membership predicate
Sun, 01 Jan 2012 11:28:45 +0100 haftmann cleanup of code declarations
Thu, 05 Jan 2012 20:26:01 +0100 wenzelm discontinued Syntax.positions -- atomic parse trees are always annotated;
Thu, 05 Jan 2012 18:18:39 +0100 wenzelm improved case syntax: more careful treatment of position constraints, which enables PIDE markup;
Thu, 05 Jan 2012 15:31:49 +0100 wenzelm misc tuning;
Thu, 05 Jan 2012 14:48:41 +0100 wenzelm prefer raw_message for protocol implementation;
Thu, 05 Jan 2012 14:34:18 +0100 wenzelm prefer raw_message for protocol implementation;
Thu, 05 Jan 2012 14:15:37 +0100 wenzelm prefer raw_message for protocol implementation;
Thu, 05 Jan 2012 13:27:50 +0100 wenzelm tuned signature;
Thu, 05 Jan 2012 13:24:29 +0100 wenzelm tuned signature -- emphasize special nature of protocol commands;
Thu, 05 Jan 2012 10:59:18 +0100 wenzelm updated version information;
Wed, 04 Jan 2012 15:41:18 +0100 wenzelm updated version information;
Wed, 04 Jan 2012 13:58:06 +0100 nipkow generalised type
Wed, 04 Jan 2012 12:09:53 +0100 blanchet improved "set" support by code inspection
Wed, 04 Jan 2012 12:09:53 +0100 blanchet remove subtlety whose justification got lost in time -- the new code is possibly less precise but sounder
Wed, 04 Jan 2012 12:09:53 +0100 blanchet tuning
Wed, 04 Jan 2012 12:09:53 +0100 blanchet handle higher-order occurrences of sets gracefully in model display
Wed, 04 Jan 2012 11:01:08 +0100 wenzelm prefer explicit version information;
Wed, 04 Jan 2012 10:47:07 +0100 blanchet more Nitpick doc updates
Wed, 04 Jan 2012 00:32:02 +0100 blanchet reenable Kodkodi in Mira now that Nitpick has been ported to 'a set constructor
Wed, 04 Jan 2012 00:30:53 +0100 blanchet reenable Kodkodi in Isatest now that Nitpick has been ported to 'a set constructor
Tue, 03 Jan 2012 23:41:59 +0100 blanchet fixed bisimilarity axiom -- avoid "insert" with wrong type
Tue, 03 Jan 2012 23:09:27 +0100 blanchet tuning
Tue, 03 Jan 2012 23:03:49 +0100 blanchet updated Nitpick docs after "set" reintroduction
Tue, 03 Jan 2012 18:33:18 +0100 blanchet no abuse of notation
Tue, 03 Jan 2012 18:33:18 +0100 blanchet always treat "unit" as a deep datatype, so that we get a good interaction with the record syntax (2.7 of the Nitpick manual)
Tue, 03 Jan 2012 18:33:18 +0100 blanchet more robust destruction of "set Collect" idiom
Tue, 03 Jan 2012 18:33:18 +0100 blanchet handle starred predicates correctly w.r.t. "set"
Tue, 03 Jan 2012 18:33:18 +0100 blanchet handle "Id" gracefully w.r.t. "set"
Tue, 03 Jan 2012 18:33:18 +0100 blanchet reintroduced 'refute' calls taken out after reintroducing the "set" constructor, and use "expect" feature
Tue, 03 Jan 2012 18:33:18 +0100 blanchet handle "set" correctly in Refute -- inspired by old code from Isabelle2007
Tue, 03 Jan 2012 18:33:18 +0100 blanchet create consts with proper "set" types
Tue, 03 Jan 2012 18:33:18 +0100 blanchet tuned Refute
Tue, 03 Jan 2012 18:33:18 +0100 blanchet lower cardinality for faster testing
Tue, 03 Jan 2012 18:33:18 +0100 blanchet simplify mem Collect
Tue, 03 Jan 2012 18:33:18 +0100 blanchet tuning
Tue, 03 Jan 2012 18:33:18 +0100 blanchet ported Minipick to "set"
Tue, 03 Jan 2012 18:33:18 +0100 blanchet fixed set extensionality code
Tue, 03 Jan 2012 18:33:18 +0100 blanchet tuned import
Tue, 03 Jan 2012 18:33:18 +0100 blanchet construct correct "set" type for wf goal
Tue, 03 Jan 2012 18:33:18 +0100 blanchet fixed Nitpick's typedef handling w.r.t. "set"
Tue, 03 Jan 2012 18:33:18 +0100 blanchet fixed type annotations
Tue, 03 Jan 2012 18:33:18 +0100 blanchet rationalized output (a bit)
Tue, 03 Jan 2012 18:33:17 +0100 blanchet fixed a few more bugs in \Nitpick's new "set" support
Tue, 03 Jan 2012 18:33:17 +0100 blanchet regenerate SMT example certificates, to reflect "set" type constructor
Tue, 03 Jan 2012 18:33:17 +0100 blanchet port part of Nitpick to "set" type constructor
Tue, 03 Jan 2012 18:33:17 +0100 blanchet reintroduced failing examples now that they work again, after reintroduction of "set"
Tue, 03 Jan 2012 18:33:17 +0100 blanchet ported mono calculus to handle "set" type constructors
Tue, 03 Jan 2012 18:33:17 +0100 blanchet fixed spurious catch-all patterns
Tue, 03 Jan 2012 13:06:03 +0100 wenzelm more benchmarks;
Mon, 02 Jan 2012 20:25:21 +0100 nipkow tuned
Mon, 02 Jan 2012 15:15:46 +0100 blanchet ported "Sets" example to "set" type constructor
Mon, 02 Jan 2012 15:08:40 +0100 blanchet ported a dozen of proofs to the "set" type constructor
Mon, 02 Jan 2012 14:45:13 +0100 blanchet reintroduced "metis" call taken out after reintroducing "set" as a constructor, and added two "metis" calls that used to be too slow
Mon, 02 Jan 2012 14:36:49 +0100 blanchet update docs to reflect "Manual_Nits"
Mon, 02 Jan 2012 14:32:20 +0100 blanchet removed special handling for set constants in relevance filter
Mon, 02 Jan 2012 14:26:57 +0100 blanchet reintroduced Sledgehammer call taken out by 9bc924006136, with some hints to guide the naive relevance filter
Mon, 02 Jan 2012 14:12:20 +0100 blanchet killed unfold_set_const option that makes no sense now that set is a type constructor again
Mon, 02 Jan 2012 11:54:21 +0100 nipkow tuned
Mon, 02 Jan 2012 11:33:50 +0100 nipkow removed unnecessary lemmas
Mon, 02 Jan 2012 10:51:28 +0100 nipkow tuned proofs
Sun, 01 Jan 2012 18:12:11 +0100 nipkow tuned var names
Sun, 01 Jan 2012 16:32:53 +0100 nipkow tuned argument order
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;
Wed, 28 Dec 2011 13:13:27 +0100 wenzelm discontinued broken macbroy5 and thus the obsolete ppc-darwin platform;
Wed, 28 Dec 2011 13:08:18 +0100 wenzelm more selective target "full" -- avoid failure of HOL-Datatype_Benchmark on 32bit platforms;
Wed, 28 Dec 2011 13:00:51 +0100 wenzelm print case syntax depending on "show_cases" configuration option;
Tue, 27 Dec 2011 15:38:45 +0100 huffman merged
Tue, 27 Dec 2011 15:37:33 +0100 huffman redefine some binary operations on integers work on abstract numerals instead of Int.Pls and Int.Min
Tue, 27 Dec 2011 13:16:22 +0100 huffman remove some uses of Int.succ and Int.pred
Tue, 27 Dec 2011 12:49:03 +0100 huffman removed unused lemmas
Tue, 27 Dec 2011 12:37:11 +0100 huffman remove redundant syntax declaration
(0) -30000 -10000 -3000 -1000 -192 +192 +1000 +3000 +10000 +30000 tip