src/HOL/GCD.thy
Mon, 09 Oct 2017 19:10:47 +0200 haftmann tuned imports
Sun, 08 Oct 2017 22:28:22 +0200 haftmann more fundamental definition of div and mod on int
Sun, 08 Oct 2017 22:28:20 +0200 haftmann avoid trivial definition
Sun, 08 Oct 2017 22:28:19 +0200 haftmann tuned proofs
Thu, 11 May 2017 16:47:53 +0200 haftmann more lemmas
Sun, 23 Apr 2017 14:53:33 +0200 haftmann include GCD as integral part of computational algebra in session HOL
Sat, 22 Apr 2017 22:01:35 +0200 wenzelm theories "GCD" and "Binomial" are already included in "Main": this avoids improper imports in applications;
Mon, 09 Jan 2017 19:13:49 +0100 haftmann gcd/lcm on finite sets
Sat, 17 Dec 2016 15:22:13 +0100 haftmann restructured matter on polynomials and normalized fractions
Mon, 17 Oct 2016 17:33:07 +0200 nipkow setprod -> prod
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, 18 Sep 2016 17:57:55 +0200 haftmann more generic algebraic lemmas
Sun, 18 Sep 2016 20:33:48 +0200 wenzelm tuned proofs;
Thu, 15 Sep 2016 11:48:20 +0200 nipkow renamed listsum -> sum_list, listprod ~> prod_list
Thu, 14 Jul 2016 11:34:18 +0200 wenzelm misc tuning and modernization;
Fri, 01 Jul 2016 08:35:15 +0200 Manuel Eberl More lemmas on Gcd/Lcm
Wed, 25 May 2016 11:49:40 +0200 wenzelm isabelle update_cartouches -c -t;
Mon, 18 Apr 2016 20:56:13 +0200 haftmann capitalized GCD and LCM syntax
Fri, 26 Feb 2016 22:15:09 +0100 Manuel Eberl Tuned Euclidean Rings/GCD rings
Wed, 17 Feb 2016 21:51:58 +0100 haftmann dropped various legacy fact bindings and tuned proofs
Wed, 17 Feb 2016 21:51:57 +0100 haftmann more sophisticated GCD syntax
Wed, 17 Feb 2016 21:51:57 +0100 haftmann cleansed junk-producing interpretations for gcd/lcm on nat altogether
Wed, 17 Feb 2016 21:51:57 +0100 haftmann dropped various legacy fact bindings
Wed, 17 Feb 2016 21:51:57 +0100 haftmann generalized some lemmas;
Wed, 17 Feb 2016 21:51:56 +0100 haftmann more theorems concerning gcd/lcm/Gcd/Lcm
Wed, 17 Feb 2016 21:51:56 +0100 haftmann further generalization and polishing
Wed, 17 Feb 2016 21:51:56 +0100 haftmann pulled out legacy aliasses and infamous dvd interpretations into theory appendix
Wed, 17 Feb 2016 21:51:56 +0100 haftmann prefer abbreviations for compound operators INFIMUM and SUPREMUM
Wed, 30 Dec 2015 11:37:29 +0100 wenzelm isabelle update_cartouches -c -t;
Mon, 28 Dec 2015 19:23:15 +0100 wenzelm more symbols;
Mon, 28 Dec 2015 01:26:34 +0100 wenzelm prefer symbols for "abs";
Thu, 24 Dec 2015 09:42:49 +0100 haftmann tuned proofs and augmented lemmas
Tue, 22 Dec 2015 15:38:59 +0100 haftmann tuned proofs and augmented some lemmas
Fri, 18 Dec 2015 11:14:28 +0100 Andreas Lochbihler add gcd instance for integer and serialisation to target language operations
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.
Mon, 09 Nov 2015 15:48:17 +0100 wenzelm qualifier is mandatory by default;
Wed, 04 Nov 2015 08:13:52 +0100 ballarin Keyword 'rewrites' identifies rewrite morphisms.
Sun, 13 Sep 2015 22:56:52 +0200 wenzelm tuned proofs -- less legacy;
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:41 +0200 haftmann more cautious use of [iff] declarations
Wed, 08 Jul 2015 14:01:41 +0200 haftmann avoid explicit definition of the relation of associated elements in a ring -- prefer explicit normalization instead
Wed, 08 Jul 2015 14:01:40 +0200 haftmann eliminated some duplication
Wed, 08 Jul 2015 14:01:39 +0200 haftmann more algebraic properties for gcd/lcm
Sat, 27 Jun 2015 20:20:33 +0200 haftmann tuned code setup
Sat, 27 Jun 2015 20:20:32 +0200 haftmann algebraic specification for set gcd
Thu, 25 Jun 2015 23:33:47 +0200 wenzelm tuned proofs;
Wed, 17 Jun 2015 23:01:19 +0200 wenzelm tuned proofs -- slightly faster;
Tue, 02 Jun 2015 09:10:05 +0200 wenzelm tuned proof;
Thu, 30 Apr 2015 15:28:01 +0100 paulson tidying some messy proofs
Wed, 08 Apr 2015 21:48:59 +0200 wenzelm eliminated hard tabs;
Wed, 25 Mar 2015 10:44:57 +0100 wenzelm prefer local fixes;
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
Sun, 15 Feb 2015 17:01:22 +0100 haftmann explicit equivalence for strict order on lattices
Tue, 10 Feb 2015 14:29:36 +0100 wenzelm indicate slow proof (approx. 20s);
Mon, 17 Nov 2014 14:55:32 +0100 haftmann formally self-contained gcd type classes
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Thu, 30 Oct 2014 21:02:01 +0100 haftmann more simp rules concerning dvd and even/odd
less more (0) -100 -60 tip