src/HOL/Int.thy
Sun, 20 Nov 2011 21:07:10 +0100 wenzelm eliminated obsolete "standard";
Thu, 17 Nov 2011 06:04:59 +0100 huffman simplify some proofs
Thu, 17 Nov 2011 06:01:47 +0100 huffman Int.thy: remove duplicate lemmas double_less_0_iff and odd_less_0, use {even,odd}_less_0_iff instead
Thu, 20 Oct 2011 17:27:14 +0200 huffman removed mult_Bit1 from int_arith_rules (cf. 882403378a41 and 3078fd2eec7b, where mult_num1 erroneously replaced mult_1)
Wed, 19 Oct 2011 15:42:43 +0200 wenzelm inlined @{thms} (ML compile-time) allows to get rid of legacy zadd_ac as well (cf. 49e305100097);
Wed, 19 Oct 2011 08:37:26 +0200 bulwahn removing old code generator setup for integers
Sun, 09 Oct 2011 11:13:53 +0200 huffman Int.thy: discontinued some legacy theorems
Sun, 04 Sep 2011 07:15:13 -0700 huffman introduce abbreviation 'int' earlier in Int.thy
Sun, 04 Sep 2011 06:27:59 -0700 huffman move lemmas nat_le_iff and nat_mono into Int.thy
Sat, 03 Sep 2011 16:00:09 -0700 huffman remove duplicate lemma nat_zero in favor of nat_0
Wed, 29 Jun 2011 18:12:34 +0200 wenzelm modernized some simproc setup;
Thu, 23 Jun 2011 09:04:20 -0700 huffman added number_semiring class, plus a few new lemmas;
Wed, 04 May 2011 15:37:39 +0200 wenzelm proper case_names for int_cases, int_of_nat_induct;
Tue, 19 Apr 2011 23:57:28 +0200 wenzelm eliminated Codegen.mode in favour of explicit argument;
Sun, 13 Mar 2011 22:55:50 +0100 wenzelm tuned headers;
Tue, 30 Nov 2010 15:58:09 +0100 haftmann adapted proofs to slightly changed definitions of congruent(2)
Fri, 01 Oct 2010 16:05:25 +0200 haftmann constant `contents` renamed to `the_elem`
Fri, 27 Aug 2010 19:34:23 +0200 haftmann renamed class/constant eq to equal; tuned some instantiations
Mon, 19 Jul 2010 16:09:44 +0200 haftmann diff_minus subsumes diff_def
Mon, 12 Jul 2010 10:48:37 +0200 haftmann dropped superfluous [code del]s
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
Mon, 10 May 2010 14:55:04 +0200 haftmann moved int induction lemma to theory Int as int_bidirectional_induct
Fri, 07 May 2010 09:51:55 +0200 haftmann moved lemma zdvd_period to theory Int
Thu, 06 May 2010 23:11:56 +0200 haftmann moved some lemmas from Groebner_Basis here
Thu, 06 May 2010 18:16:07 +0200 haftmann moved generic lemmas to appropriate places
Tue, 27 Apr 2010 12:20:09 +0200 haftmann got rid of [simplified]
Mon, 26 Apr 2010 15:37:50 +0200 haftmann use new classes (linordered_)field_inverse_zero
Mon, 26 Apr 2010 11:34:17 +0200 haftmann class division_ring_inverse_zero
Fri, 16 Apr 2010 21:28:09 +0200 wenzelm replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
Tue, 06 Apr 2010 10:46:28 +0200 boehmes added missing mult_1_left to linarith simp rules
Thu, 18 Mar 2010 13:14:54 +0100 blanchet merged
Thu, 18 Mar 2010 12:58:52 +0100 blanchet now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
Wed, 17 Mar 2010 19:55:07 +0100 boehmes tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
Sun, 07 Mar 2010 08:40:38 -0800 huffman add more simp rules for Ints
Thu, 18 Feb 2010 14:21:44 -0800 huffman get rid of many duplicate simp rule warnings
Sat, 13 Feb 2010 23:24:57 +0100 wenzelm modernized structures;
Mon, 08 Feb 2010 17:12:38 +0100 haftmann renamed OrderedGroup to Groups; split theory Ring_and_Field into Rings Fields
Mon, 08 Feb 2010 14:06:41 +0100 haftmann separate library theory for type classes combining lattices with various algebraic structures
Fri, 05 Feb 2010 14:33:50 +0100 haftmann more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
Thu, 10 Dec 2009 17:34:18 +0000 paulson streamlined proofs
Fri, 13 Nov 2009 14:14:04 +0100 nipkow renamed lemmas "anti_sym" -> "antisym"
Sun, 08 Nov 2009 19:15:37 +0100 wenzelm modernized structure Reorient_Proc;
Fri, 30 Oct 2009 18:32:40 +0100 haftmann tuned code setup
Thu, 29 Oct 2009 22:13:11 +0100 haftmann moved some dvd [int] facts to Int
Thu, 29 Oct 2009 11:41:38 +0100 haftmann moved some dvd [int] facts to Int
Wed, 28 Oct 2009 19:09:47 +0100 haftmann moved theory Divides after theory Nat_Numeral; tuned some proof texts
Wed, 21 Oct 2009 17:34:35 +0200 blanchet renamed "nitpick_const_xxx" attributes to "nitpick_xxx" and "nitpick_ind_intros" to "nitpick_intros"
Fri, 28 Aug 2009 19:15:59 +0200 nipkow tuned proofs
Wed, 29 Jul 2009 16:42:47 +0200 haftmann added numeral code postprocessor rules on type int
Tue, 14 Jul 2009 16:27:32 +0200 haftmann prefer code_inline over code_unfold; use code_unfold_post where appropriate
Tue, 14 Jul 2009 10:54:04 +0200 haftmann code attributes use common underscore convention
Mon, 11 May 2009 15:18:32 +0200 haftmann tuned interface of Lin_Arith
Fri, 08 May 2009 09:48:07 +0200 haftmann modules numeral_simprocs, nat_numeral_simprocs; proper structures for numeral simprocs
Fri, 08 May 2009 08:00:11 +0200 haftmann moved int_factor_simprocs.ML to theory Int
Wed, 29 Apr 2009 17:15:01 -0700 huffman reimplement reorientation simproc using theory data
Wed, 29 Apr 2009 14:20:26 +0200 haftmann farewell to class recpower
Tue, 28 Apr 2009 15:50:29 +0200 haftmann reorganization of power lemmas
Tue, 28 Apr 2009 13:34:46 +0200 haftmann local syntax for Ints; ephermal re-globalization
Mon, 27 Apr 2009 10:11:44 +0200 haftmann cleaned up theory power further
Wed, 22 Apr 2009 19:09:21 +0200 haftmann power operation defined generic
less more (0) -100 -60 tip