src/HOL/Divides.thy
Fri, 19 Jun 2015 07:53:33 +0200 haftmann generalized some theorems about integral domains and moved to HOL theories
Fri, 12 Jun 2015 08:53:23 +0200 haftmann uniform _ div _ as infix syntax for ring division
Mon, 01 Jun 2015 18:59:22 +0200 haftmann implicit partial divison operation in integral domains
Mon, 01 Jun 2015 18:59:21 +0200 haftmann separate class for division operator, with particular syntax added in more specific classes
Sat, 28 Mar 2015 21:32:48 +0100 haftmann clarified no_zero_devisors: makes only sense in a semiring;
Mon, 23 Mar 2015 19:05:14 +0100 haftmann distributivity of partial minus establishes desired properties of dvd in semirings
Wed, 25 Mar 2015 10:44:57 +0100 wenzelm prefer local fixes;
Wed, 18 Feb 2015 22:46:48 +0100 haftmann eliminated technical fact alias
Fri, 30 Jan 2015 17:35:03 +0100 nipkow canonical name
Fri, 16 Jan 2015 20:06:39 +0100 nipkow added simp lemma
Wed, 26 Nov 2014 20:05:34 +0100 wenzelm renamed "pairself" to "apply2", in accordance to @{apply 2};
Mon, 17 Nov 2014 14:55:33 +0100 haftmann generalized lemmas (particularly concerning dvd) as far as appropriate
Thu, 13 Nov 2014 17:19:52 +0100 hoelzl import general theorems from AFP/Markov_Models
Sun, 09 Nov 2014 10:03:17 +0100 haftmann self-contained simp rules for dvd on numerals
Wed, 05 Nov 2014 20:59:24 +0100 haftmann proper oriented equivalence of dvd predicate and mod
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Fri, 31 Oct 2014 16:56:23 +0100 wenzelm avoid noise (cf. 03ff4d1e6784);
Thu, 30 Oct 2014 21:02:01 +0100 haftmann more simp rules concerning dvd and even/odd
Sat, 25 Oct 2014 19:20:28 +0200 haftmann more simp rules;
Thu, 23 Oct 2014 19:40:41 +0200 haftmann even further downshift of theory Parity in the hierarchy
Mon, 20 Oct 2014 07:45:58 +0200 haftmann augmented and tuned facts on even/odd and division
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
less more (0) -100 -60 tip