src/HOL/Word/Word.thy
Mon, 23 Dec 2013 14:24:22 +0100 haftmann dropped redundant lemma
Mon, 23 Dec 2013 14:24:21 +0100 haftmann syntactically tuned
Mon, 23 Dec 2013 14:24:20 +0100 haftmann prefer plain bool over dedicated type for binary digits
Sat, 14 Dec 2013 20:46:36 +0100 wenzelm more antiquotations;
Sat, 14 Dec 2013 17:28:05 +0100 wenzelm proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
Tue, 19 Nov 2013 10:05:53 +0100 haftmann eliminiated neg_numeral in favour of - (numeral _)
Thu, 31 Oct 2013 11:44:20 +0100 haftmann generalized of_bool conversion
Thu, 31 Oct 2013 11:44:20 +0100 haftmann separated bit operations on type bit from generic syntactic bit operations
Thu, 31 Oct 2013 11:44:20 +0100 haftmann more lemmas on division
Sun, 18 Aug 2013 23:37:38 +0200 wenzelm tuned;
Sun, 18 Aug 2013 15:29:50 +0200 haftmann some vague grouping of related theorems, with slight tuning of headings and sorting out of dubious lemmas into separate theory
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Fri, 08 Mar 2013 13:21:06 +0100 kuncar patch Isabelle ditribution to conform to changes regarding the parametricity
Tue, 26 Feb 2013 20:09:25 +0100 wenzelm tuned;
Fri, 15 Feb 2013 08:31:31 +0100 haftmann two target language numeral types: integer and natural, as replacement for code_numeral;
Fri, 12 Oct 2012 18:58:20 +0200 wenzelm discontinued obsolete typedef (open) syntax;
Wed, 22 Aug 2012 22:55:41 +0200 wenzelm prefer ML_file over old uses;
Thu, 05 Jul 2012 17:18:55 +0200 wenzelm explicit is better than implicit;
Fri, 18 May 2012 15:08:08 +0200 kuncar don't generate code in Word because it breaks the current code setup
Thu, 19 Apr 2012 19:32:30 +0200 huffman add code lemmas for word operations
Tue, 17 Apr 2012 16:21:47 +1000 Thomas Sewell New tactic "word_bitwise" expands word equalities/inequalities into logic.
Wed, 18 Apr 2012 23:57:44 +0200 kuncar setup_lifting: no_code switch and supoport for quotient theorems
Tue, 17 Apr 2012 19:16:13 +0200 kuncar tuned the setup of lifting; generate transfer rules for typedef and Quotient thms
Fri, 06 Apr 2012 14:40:00 +0200 huffman remove now-unnecessary type annotations from lift_definition commands
Thu, 05 Apr 2012 16:25:59 +0200 huffman use standard quotient lemmas to generate transfer rules
Thu, 05 Apr 2012 14:14:16 +0200 huffman set up and use lift_definition for word operations
Thu, 05 Apr 2012 10:48:46 +0200 huffman configure transfer method for 'a word -> int
Tue, 27 Mar 2012 21:48:26 +0200 huffman mark some duplicate lemmas for deletion
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
Fri, 16 Mar 2012 15:51:53 +0100 huffman make more word theorems respect int/bin distinction
Fri, 24 Feb 2012 17:21:24 +0100 huffman remove ill-formed lemmas word_0_wi_Pls and word_m1_wi_Min
Fri, 24 Feb 2012 16:55:29 +0100 huffman avoid using Int.succ or Int.pred in proofs
Fri, 24 Feb 2012 13:50:37 +0100 huffman avoid using Int.Pls_def in proofs
Fri, 24 Feb 2012 13:37:23 +0100 huffman remove ill-formed lemmas word_pred_0_Min and word_m1_Min
Fri, 24 Feb 2012 13:33:03 +0100 huffman remove ill-formed lemma of_bl_no; adapt proofs
Fri, 24 Feb 2012 13:25:21 +0100 huffman adapt lemma mask_lem to respect int/bin distinction
Thu, 23 Feb 2012 16:09:16 +0100 huffman make more simp rules respect int/bin distinction
Thu, 23 Feb 2012 15:37:42 +0100 huffman make bool list functions respect int/bin distinction
Thu, 23 Feb 2012 13:16:18 +0100 huffman make uses of bin_sign respect int/bin distinction
Thu, 23 Feb 2012 12:45:00 +0100 huffman removed unnecessary lemma zero_bintrunc
Thu, 23 Feb 2012 12:24:34 +0100 huffman remove unnecessary lemmas
Wed, 08 Feb 2012 01:49:33 +0100 blanchet use 'primrec' to define "rotate1", for uniformity (and to help first-order tools that rely on "Spec_Rules")
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
Fri, 06 Jan 2012 16:42:15 +0100 wenzelm recovered case syntax for of_int, also with source positions (appears to be unused nonetheless);
Thu, 05 Jan 2012 15:31:49 +0100 wenzelm misc tuning;
Fri, 30 Dec 2011 16:08:35 +0100 huffman add simp rules for bitwise word operations with 1
Fri, 30 Dec 2011 11:11:57 +0100 huffman remove unnecessary intermediate lemmas
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: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 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";
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:37:11 +0100 huffman remove redundant syntax declaration
Tue, 27 Dec 2011 11:38:55 +0100 huffman declare word_of_int_{0,1} [simp], for consistency with word_of_int_bin
Fri, 23 Dec 2011 16:37:27 +0100 huffman simplify some proofs
Fri, 23 Dec 2011 15:55:23 +0100 huffman remove redundant lemma word_sub_def
Fri, 23 Dec 2011 11:50:12 +0100 huffman remove two conflicting simp rules for 'number_of (number_of _)' pattern
Wed, 14 Dec 2011 08:32:48 +0100 huffman replace 'lemmas' with 'lemma'
Tue, 13 Dec 2011 12:36:41 +0100 huffman towards removing BIT_simps from the simpset
Mon, 12 Dec 2011 08:19:37 +0100 huffman replace more uses of 'lemmas' with explicit 'lemma';
Sun, 11 Dec 2011 09:55:57 +0100 huffman replace many uses of 'lemmas' with 'lemma';
Sat, 10 Dec 2011 22:00:42 +0100 huffman prove class instances without extra lemmas
Sat, 10 Dec 2011 21:48:16 +0100 huffman finite class instance for word type; remove unused lemmas
Sat, 10 Dec 2011 21:07:59 +0100 huffman remove unused lemmas
Sat, 10 Dec 2011 16:24:22 +0100 huffman generalize some lemmas
Sat, 10 Dec 2011 08:29:19 +0100 huffman tidied Word.thy;
Fri, 09 Dec 2011 14:52:51 +0100 huffman remove redundant lemma word_diff_minus
Wed, 30 Nov 2011 16:27:10 +0100 wenzelm prefer typedef without extra definition and alternative name;
Wed, 23 Nov 2011 22:59:39 +0100 wenzelm modernized some old-style infix operations, which were left over from the time of ML proof scripts;
Sun, 20 Nov 2011 20:59:30 +0100 wenzelm eliminated obsolete "standard";
Fri, 18 Nov 2011 06:50:05 +0100 huffman Word.thy: reduce usage of numeral-representation-dependent thms like number_of_is_id in proofs
Fri, 18 Nov 2011 04:56:35 +0100 huffman merged
Thu, 17 Nov 2011 15:07:46 +0100 huffman HOL-Word: removed more duplicate theorems
Thu, 17 Nov 2011 14:52:05 +0100 huffman HOL-Word: removed many duplicate theorems (see NEWS)
Thu, 17 Nov 2011 14:24:10 +0100 huffman Word.thy: rearrange to instantiate arithmetic classes together with arithmetic operations
Thu, 17 Nov 2011 12:38:03 +0100 huffman move definitions of bitwise operators into appropriate document section
Thu, 17 Nov 2011 21:58:10 +0100 wenzelm eliminated slightly odd Rep' with dynamically-scoped [simplified];
Wed, 16 Nov 2011 13:58:31 +0100 huffman remove redundant lemmas bin_last_mod and bin_rest_div, use bin_last_def and bin_rest_def instead
Wed, 16 Nov 2011 12:29:50 +0100 huffman simplify proof of word_of_int; remove several now-unused lemmas about Rep_Integ
Fri, 28 Oct 2011 11:02:27 +0200 huffman use simproc_setup for cancellation simprocs, to get proper name bindings
Fri, 16 Sep 2011 12:10:15 +1000 kleing removed word_neq_0_conv from simpset, it's almost never wanted.
Mon, 12 Sep 2011 07:55:43 +0200 nipkow new fastforce replacing fastsimp - less confusing name
Wed, 07 Sep 2011 09:02:58 -0700 huffman avoid using legacy theorem names
Wed, 07 Sep 2011 00:08:09 +0200 wenzelm tuned proofs;
Fri, 13 May 2011 22:55:00 +0200 wenzelm proper Proof.context for classical tactics;
Fri, 14 Jan 2011 15:44:47 +0100 wenzelm eliminated global prems;
Wed, 29 Dec 2010 17:34:41 +0100 wenzelm explicit file specifications -- avoid secondary load path;
Tue, 07 Dec 2010 14:53:44 +0100 boehmes moved smt_word.ML into the directory of the Word library
Tue, 30 Nov 2010 20:52:49 +0100 haftmann code preprocessor setup for numerals on word type;
Fri, 01 Oct 2010 16:05:25 +0200 haftmann constant `contents` renamed to `the_elem`
Mon, 13 Sep 2010 11:13:15 +0200 nipkow renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
Tue, 07 Sep 2010 10:05:19 +0200 nipkow expand_fun_eq -> ext_iff
Fri, 27 Aug 2010 19:34:23 +0200 haftmann renamed class/constant eq to equal; tuned some instantiations
Wed, 18 Aug 2010 14:55:10 +0200 haftmann moved spurious auxiliary lemma here
Mon, 19 Jul 2010 16:09:44 +0200 haftmann diff_minus subsumes diff_def
Fri, 09 Jul 2010 08:11:10 +0200 haftmann nicer xsymbol syntax for fcomp and scomp
Thu, 01 Jul 2010 13:32:14 +0200 haftmann avoid bitstrings in generated code
Wed, 30 Jun 2010 17:12:38 +0200 haftmann one unified Word theory
Wed, 12 May 2010 23:54:04 +0200 boehmes layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
Mon, 08 Feb 2010 17:12:32 +0100 haftmann tuned spelling
Mon, 26 Jan 2009 22:14:16 +0100 haftmann entry point for Word library now named Word
less more (0) tip