src/HOL/Divides.thy
Fri, 14 Jun 2019 08:34:27 +0000 haftmann slightly more specialized name for type class
Mon, 04 Feb 2019 12:16:03 +0100 Manuel Eberl More material for HOL-Number_Theory: ord, Carmichael's function, primitive roots
Sat, 19 Jan 2019 20:40:17 +0000 haftmann algebraized more material from theory Divides
Fri, 04 Jan 2019 23:22:53 +0100 wenzelm isabelle update -u control_cartouches;
Wed, 31 Oct 2018 15:53:32 +0100 wenzelm clarified ML_Context.expression: it is a closed expression, not a let-declaration -- thus source positions are more accurate (amending d8849cfad60f, 162a4c2e97bc);
Mon, 16 Jul 2018 23:33:28 +0100 paulson de-applying and simplifying proofs
Sat, 14 Jul 2018 22:32:15 +0100 paulson de-applying
Fri, 13 Jul 2018 17:18:07 +0100 paulson de-applying
Thu, 24 May 2018 09:18:29 +0200 haftmann avoid overaggressive classical rule
Wed, 23 May 2018 07:13:11 +0000 haftmann grouped material on numeral division
Sat, 12 May 2018 22:20:46 +0200 haftmann removed some non-essential rules
Sun, 06 May 2018 18:20:25 +0000 haftmann removed some lemma duplicates
Mon, 12 Mar 2018 08:25:35 +0000 haftmann eliminiated superfluous class semiring_bits
Sat, 10 Mar 2018 19:36:59 +0000 haftmann abstract algebraic bit operations
Tue, 19 Dec 2017 13:58:12 +0100 wenzelm isabelle update_cartouches -c -t;
Sat, 02 Dec 2017 16:50:53 +0000 haftmann more simplification rules
Sun, 26 Nov 2017 21:08:32 +0100 wenzelm more symbols;
Thu, 23 Nov 2017 13:00:00 +0000 haftmann new simp rule
Fri, 20 Oct 2017 07:46:10 +0200 haftmann added lemmas and tuned proofs
Mon, 09 Oct 2017 19:10:48 +0200 haftmann tuned proofs
Sun, 08 Oct 2017 22:28:22 +0200 haftmann euclidean rings need no normalization
Sun, 08 Oct 2017 22:28:22 +0200 haftmann more fundamental definition of div and mod on int
Sun, 08 Oct 2017 22:28:22 +0200 haftmann one uniform type class for parity structures
Sun, 08 Oct 2017 22:28:22 +0200 haftmann generalized some rules
Sun, 08 Oct 2017 22:28:21 +0200 haftmann generalized simproc
Sun, 08 Oct 2017 22:28:21 +0200 haftmann elementary definition of division on natural numbers
Sun, 08 Oct 2017 22:28:21 +0200 haftmann abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
Sun, 08 Oct 2017 22:28:20 +0200 haftmann avoid fact name clashes
Sun, 08 Oct 2017 22:28:19 +0200 haftmann spelling and tuned whitespace
Fri, 08 Sep 2017 00:02:33 +0200 blanchet speed up proofs slightly
Sun, 23 Apr 2017 14:53:35 +0200 haftmann more lemmas
Mon, 09 Jan 2017 18:53:06 +0100 haftmann slightly generalized type class hierarchy concerning unit factors, to allow for lean polynomial normalization
Wed, 04 Jan 2017 21:28:29 +0100 haftmann moved euclidean ring to HOL
Sat, 31 Dec 2016 08:12:31 +0100 haftmann more elementary rules about div / mod on int
Thu, 22 Dec 2016 10:42:08 +0100 haftmann more uniform div/mod relations
Tue, 20 Dec 2016 15:39:13 +0100 haftmann emphasize dedicated rewrite rules for congruences
Sat, 17 Dec 2016 15:22:14 +0100 haftmann reoriented congruence rules in non-explosive direction
Sat, 17 Dec 2016 15:22:14 +0100 haftmann more fine-grained type class hierarchy for div and mod
Sun, 16 Oct 2016 13:47:37 +0200 haftmann clarified prover-specific rules
Sun, 16 Oct 2016 09:31:06 +0200 haftmann eliminated irregular aliasses
Sun, 16 Oct 2016 09:31:05 +0200 haftmann clarified theorem names
Sun, 16 Oct 2016 09:31:05 +0200 haftmann eliminated irregular aliasses
Sun, 16 Oct 2016 09:31:05 +0200 haftmann more standardized theorem names for facts involving the div and mod identity
Sun, 16 Oct 2016 09:31:04 +0200 haftmann more standardized names
Sun, 16 Oct 2016 09:31:03 +0200 haftmann de-orphanized declaration
Wed, 12 Oct 2016 20:38:47 +0200 haftmann separate type class for arbitrary quotient and remainder partitions
Mon, 03 Oct 2016 14:34:32 +0200 haftmann more lemmas
Mon, 26 Sep 2016 07:56:54 +0200 haftmann syntactic type class for operation mod named after mod;
Mon, 26 Sep 2016 07:56:54 +0200 haftmann more lemmas
Sun, 11 Sep 2016 00:14:44 +0200 wenzelm tuned proofs;
Thu, 14 Jul 2016 14:43:09 +0200 eberlm Tuned looping simp rules in semiring_div
Sat, 09 Jul 2016 13:26:16 +0200 haftmann more lemmas to emphasize {0::nat..(<)n} as canonical representation of intervals on nat
Thu, 16 Jun 2016 17:57:09 +0200 eberlm Various additions to polynomials, FPSs, Gamma function
Wed, 25 May 2016 11:49:40 +0200 wenzelm isabelle update_cartouches -c -t;
Mon, 25 Apr 2016 16:09:26 +0200 wenzelm eliminated old 'def';
Sat, 12 Mar 2016 22:04:52 +0100 haftmann model characters directly as range 0..255
Tue, 23 Feb 2016 16:25:08 +0100 nipkow more canonical names
Mon, 28 Dec 2015 01:26:34 +0100 wenzelm prefer symbols for "abs";
Mon, 07 Dec 2015 10:38:04 +0100 wenzelm isabelle update_cartouches -c -t;
Fri, 13 Nov 2015 12:27:13 +0000 paulson Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
Sat, 17 Oct 2015 13:18:43 +0200 haftmann qualify some names stemming from internal bootstrap constructions
Sun, 27 Sep 2015 10:11:15 +0200 haftmann monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
Sat, 19 Sep 2015 22:32:26 +0200 wenzelm eliminated suspicious unicode;
Tue, 01 Sep 2015 22:32:58 +0200 wenzelm eliminated \<Colon>;
Thu, 13 Aug 2015 15:22:11 +0200 haftmann qualified adjust_*
Sat, 08 Aug 2015 10:51:33 +0200 haftmann direct bootstrap of integer division from natural division
Thu, 06 Aug 2015 23:56:48 +0200 haftmann slight cleanup of lemmas
Sat, 18 Jul 2015 22:58:50 +0200 wenzelm isabelle update_cartouches;
Wed, 08 Jul 2015 20:19:12 +0200 haftmann tuned facts
Wed, 08 Jul 2015 14:01:34 +0200 haftmann moved normalization and unit_factor into Main HOL corpus
Tue, 23 Jun 2015 16:55:28 +0100 paulson Amalgamation of the class comm_semiring_1_diff_distrib into comm_semiring_1_cancel. Moving axiom le_add_diff_inverse2 from semiring_numeral_div to linordered_semidom.
Fri, 19 Jun 2015 07:53:35 +0200 haftmann separate class for notions specific for integral (semi)domains, in contrast to fields where these are trivial
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);
less more (0) -120 tip