src/HOL/Int.thy
Tue, 10 Mar 2015 15:20:40 +0000 paulson Removal of the file HOL/Number_Theory/Binomial!! And class field_char_0 now declared in Int.thy
Thu, 05 Mar 2015 17:30:29 +0000 paulson The function frac. Various lemmas about limits, series, the exp function, etc.
Wed, 04 Mar 2015 19:53:18 +0100 wenzelm tuned signature -- prefer qualified names;
Wed, 18 Feb 2015 22:46:48 +0100 haftmann eliminated technical fact alias
Sat, 14 Feb 2015 10:24:15 +0100 haftmann dropped redundancy
Thu, 13 Nov 2014 17:19:52 +0100 hoelzl import general theorems from AFP/Markov_Models
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Sun, 12 Oct 2014 17:05:35 +0200 haftmann some more facts on divisibility
Sun, 12 Oct 2014 17:05:34 +0200 haftmann generalized and consolidated some theorems concerning divisibility
Thu, 02 Oct 2014 11:33:06 +0200 haftmann moved lemmas out of Int.thy which have nothing to do with int
Sat, 05 Jul 2014 11:01:53 +0200 haftmann prefer ac_simps collections over separate name bindings for add and mult
Fri, 04 Jul 2014 20:18:47 +0200 haftmann reduced name variants for assoc and commute on plus and mult
Wed, 07 May 2014 12:25:35 +0200 hoelzl avoid the Complex constructor, use the more natural Re/Im view; moved csqrt to Complex.
Thu, 10 Apr 2014 17:48:32 +0200 kuncar simplify and fix theories thanks to 356a5efdb278
Thu, 06 Mar 2014 15:40:33 +0100 blanchet renamed 'fun_rel' to 'rel_fun'
Tue, 04 Mar 2014 15:26:12 -0800 huffman remove simp rules made redundant by the replacement of neg_numeral with negated numerals
Wed, 12 Feb 2014 08:35:56 +0100 blanchet transformed 'option' and 'list' into new-style datatypes (but register them as old-style as well)
Tue, 21 Jan 2014 13:21:55 +0100 traytel removed theory dependency of BNF_LFP on Datatype
Mon, 20 Jan 2014 21:32:41 +0100 blanchet moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
Wed, 25 Dec 2013 17:39:06 +0100 haftmann prefer more canonical names for lemmas on min/max
Tue, 19 Nov 2013 10:05:53 +0100 haftmann eliminiated neg_numeral in favour of - (numeral _)
Mon, 04 Nov 2013 20:10:06 +0100 haftmann streamlined setup of linear arithmetic
Fri, 01 Nov 2013 18:51:14 +0100 haftmann more simplification rules on unary and binary minus
Thu, 31 Oct 2013 11:44:20 +0100 haftmann restructed
Fri, 18 Oct 2013 10:43:20 +0200 blanchet killed most "no_atp", to make Sledgehammer more complete
Mon, 16 Sep 2013 15:30:20 +0200 kuncar use lifting_forget for deregistering numeric types as a quotient type
Sun, 18 Aug 2013 15:29:50 +0200 haftmann added lemma
Sun, 23 Jun 2013 21:16:07 +0200 haftmann migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
Wed, 15 May 2013 12:10:39 +0200 kuncar stronger reflexivity prover
Wed, 20 Feb 2013 12:04:42 +0100 hoelzl split dense into inner_dense_order and no_top/no_bot
Tue, 19 Feb 2013 15:03:36 +0100 kuncar delete also predicates on relations when hiding an implementation of an abstract type
Fri, 15 Feb 2013 08:31:31 +0100 haftmann two target language numeral types: integer and natural, as replacement for code_numeral;
Thu, 14 Feb 2013 12:24:42 +0100 haftmann abandoned theory Plain
Fri, 19 Oct 2012 15:12:52 +0200 webertj Renamed {left,right}_distrib to distrib_{right,left}.
Wed, 22 Aug 2012 22:55:41 +0200 wenzelm prefer ML_file over old uses;
Sat, 02 Jun 2012 08:27:29 +0200 huffman transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
Wed, 30 May 2012 16:59:20 +0200 huffman convert Int.thy to use lifting and transfer
Wed, 30 May 2012 14:55:44 +0200 huffman remove unnecessary simp rules involving Abs_Integ
Sun, 01 Apr 2012 16:09:58 +0200 huffman removed Nat_Numeral.thy, moving all theorems elsewhere
Fri, 30 Mar 2012 16:44:23 +0200 huffman load Tools/numeral.ML in Num.thy
Fri, 30 Mar 2012 15:56:12 +0200 huffman set up numeral reorient simproc in Num.thy
Fri, 30 Mar 2012 08:10:28 +0200 huffman move lemmas from Nat_Numeral to Int.thy and Num.thy
Thu, 29 Mar 2012 14:09:10 +0200 huffman move many lemmas from Nat_Numeral.thy to Power.thy or Num.thy
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
Fri, 02 Mar 2012 09:35:32 +0100 bulwahn adding finiteness of intervals on integer sets; adding another finiteness theorem for multisets
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
Wed, 30 Nov 2011 16:27:10 +0100 wenzelm prefer typedef without extra definition and alternative name;
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;
less more (0) -100 -60 tip