src/HOL/Divides.thy
Fri, 10 Oct 2014 19:55:32 +0200 haftmann specialized specification: avoid trivial instances
Thu, 02 Oct 2014 11:33:05 +0200 haftmann redundant: dropped
Sun, 21 Sep 2014 16:56:11 +0200 haftmann explicit separation of signed and unsigned numerals using existing lexical categories num and xnum
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, 11 Jun 2014 14:24:23 +1000 Thomas Sewell Hypsubst preserves equality hypotheses
Wed, 12 Feb 2014 14:32:45 +0100 wenzelm merged, resolving some conflicts;
Wed, 12 Feb 2014 13:56:43 +0100 wenzelm eliminated hard tabs (assuming tab-width=2);
Wed, 12 Feb 2014 08:35:57 +0100 blanchet renamed '{prod,sum,bool,unit}_case' to 'case_...'
Thu, 30 Jan 2014 10:00:53 +0100 haftmann more direct simplification rules for 1 div/mod numeral;
Mon, 20 Jan 2014 21:32:41 +0100 blanchet moved 'fundef_cong' attribute (and other basic 'fun' stuff) up the dependency chain
Tue, 19 Nov 2013 10:05:53 +0100 haftmann eliminiated neg_numeral in favour of - (numeral _)
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 moving generic lemmas out of theory parity, disregarding some unused auxiliary lemmas;
Thu, 31 Oct 2013 11:44:20 +0100 haftmann explicit type class for modelling even/odd parity
Thu, 31 Oct 2013 11:44:20 +0100 haftmann more lemmas on division
Tue, 03 Sep 2013 01:12:40 +0200 wenzelm tuned proofs -- clarified flow of facts wrt. calculation;
Mon, 26 Aug 2013 11:41:17 +0200 wenzelm removed junk;
Sun, 18 Aug 2013 15:35:01 +0200 haftmann spelling and typos
Sun, 18 Aug 2013 15:29:50 +0200 haftmann execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
Sun, 18 Aug 2013 15:29:50 +0200 haftmann relaxed preconditions
Sun, 18 Aug 2013 15:29:50 +0200 haftmann type class for generic division algorithm on numerals
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, 19 Jun 2013 17:34:56 +0200 noschinl added lemma
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Thu, 28 Feb 2013 11:40:23 +0100 wenzelm proper place for cancel_div_mod.ML (see also ee729dbd1b7f and ec7f10155389);
Sun, 17 Feb 2013 21:29:30 +0100 haftmann Sieve of Eratosthenes
Fri, 07 Dec 2012 16:25:33 +0100 wenzelm avoid ML_file in large theory files to improve performance of dependency discovery of main HOL (approx. 1s CPU time) -- relevant for any application using it, e.g. small paper sessions;
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;
Fri, 27 Jul 2012 19:27:21 +0200 huffman move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
Mon, 02 Apr 2012 09:18:16 +0200 huffman add simp rules for dvd on negative numerals
Sun, 01 Apr 2012 16:09:58 +0200 huffman removed Nat_Numeral.thy, moving all theorems elsewhere
Fri, 30 Mar 2012 11:16:35 +0200 huffman removed redundant nat-specific copies of theorems
Tue, 27 Mar 2012 20:19:23 +0200 huffman remove more redundant lemmas
Tue, 27 Mar 2012 16:49:23 +0200 huffman tuned proofs
Tue, 27 Mar 2012 19:21:05 +0200 huffman remove redundant lemmas
Tue, 27 Mar 2012 16:04:51 +0200 huffman generalized lemma zpower_zmod
Tue, 27 Mar 2012 15:53:48 +0200 huffman remove redundant lemma
Tue, 27 Mar 2012 15:40:11 +0200 huffman remove redundant lemma
Tue, 27 Mar 2012 15:34:04 +0200 huffman generalize more div/mod lemmas
Tue, 27 Mar 2012 15:27:49 +0200 huffman generalize some theorems about div/mod
Tue, 27 Mar 2012 14:49:56 +0200 huffman remove redundant lemmas
Tue, 27 Mar 2012 12:42:54 +0200 huffman move int::ring_div instance upward, simplify several proofs
Tue, 27 Mar 2012 11:45:02 +0200 huffman rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
Tue, 27 Mar 2012 11:41:16 +0200 huffman extend definition of divmod_int_rel to handle denominator=0 case
Tue, 27 Mar 2012 11:02:18 +0200 huffman tuned proofs
Tue, 27 Mar 2012 10:34:12 +0200 huffman shorten a proof
Tue, 27 Mar 2012 10:20:31 +0200 huffman simplify some proofs
Tue, 27 Mar 2012 09:54:39 +0200 huffman rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
Tue, 27 Mar 2012 09:44:56 +0200 huffman simplify some proofs
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
Tue, 21 Feb 2012 11:04:38 +0100 huffman remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
Mon, 20 Feb 2012 15:17:03 +0100 bulwahn removing some unnecessary premises from Divides
Mon, 20 Feb 2012 14:23:46 +0100 huffman simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
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
Sun, 20 Nov 2011 21:07:10 +0100 wenzelm eliminated obsolete "standard";
Wed, 16 Nov 2011 15:20:27 +0100 huffman rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
Fri, 21 Oct 2011 11:17:14 +0200 bulwahn replacing code_inline by code_unfold, removing obsolete code_unfold, code_inline del now that the ancient code generator is removed
less more (0) -100 -60 tip