src/HOL/Library/Formal_Power_Series.thy
Tue, 05 Nov 2013 09:45:02 +0100 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
Fri, 01 Nov 2013 18:51:14 +0100 more simplification rules on unary and binary minus
Tue, 03 Sep 2013 01:12:40 +0200 tuned proofs -- clarified flow of facts wrt. calculation;
Sun, 25 Aug 2013 23:20:25 +0200 tuned proofs;
Sun, 25 Aug 2013 21:25:17 +0200 tuned proofs;
Sun, 18 Aug 2013 19:59:19 +0200 more symbols;
Wed, 07 Aug 2013 23:20:11 +0200 tuned proofs;
Wed, 07 Aug 2013 21:16:20 +0200 tuned proofs;
Wed, 07 Aug 2013 14:47:50 +0200 tuned proofs;
Tue, 26 Mar 2013 20:02:02 +0100 tuned imports;
Sat, 23 Mar 2013 20:50:39 +0100 fundamental revision of big operators on sets
Wed, 13 Feb 2013 16:35:07 +0100 complete metric for formal power series
Fri, 19 Oct 2012 15:12:52 +0200 Renamed {left,right}_distrib to distrib_{right,left}.
Fri, 12 Oct 2012 18:58:20 +0200 discontinued obsolete typedef (open) syntax;
Fri, 10 Aug 2012 16:19:51 +0200 tuned proofs;
Fri, 30 Mar 2012 11:16:35 +0200 removed redundant nat-specific copies of theorems
Sun, 25 Mar 2012 20:15:39 +0200 merged fork with new numeral representation (see NEWS)
Fri, 02 Mar 2012 09:35:33 +0100 removing finiteness goals
Fri, 06 Jan 2012 10:19:48 +0100 prefer listsum over foldl plus 0
Fri, 12 Aug 2011 14:45:50 -0700 make more HOL theories work with separate set type
Sun, 13 Mar 2011 22:55:50 +0100 tuned headers;
Mon, 13 Sep 2010 11:13:15 +0200 renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
Tue, 07 Sep 2010 10:05:19 +0200 expand_fun_eq -> ext_iff
Tue, 08 Jun 2010 16:37:22 +0200 tuned quotes, antiquotations and whitespace
Tue, 11 May 2010 08:36:02 +0200 renamed former Int.int_induct to Int.int_of_nat_induct, former Presburger.int_induct to Int.int_induct: is more conservative and more natural than the intermediate solution
Tue, 11 May 2010 08:29:42 +0200 theorem Presburger.int_induct has been renamed to Int.int_bidirectional_induct
Mon, 26 Apr 2010 15:37:50 +0200 use new classes (linordered_)field_inverse_zero
Mon, 26 Apr 2010 11:34:19 +0200 dropped group_simps, ring_simps, field_eq_simps
Fri, 23 Apr 2010 16:38:51 +0200 epheremal replacement of field_simps by field_eq_simps; dropped old division_by_zero instance
Fri, 23 Apr 2010 16:17:25 +0200 epheremal replacement of field_simps by field_eq_simps
Wed, 17 Feb 2010 10:30:36 -0800 fix more looping simp rules
Sat, 17 Oct 2009 14:43:18 +0200 eliminated hard tabulators, guessing at each author's individual tab-width;
Mon, 31 Aug 2009 14:09:42 +0200 tuned the simp rules for Int involving insert and intervals.
Wed, 26 Aug 2009 17:38:02 +0100 merged
Tue, 19 May 2009 14:13:37 +0100 merged
Tue, 19 May 2009 14:13:23 +0100 Derivative of general reverses
Thu, 23 Jul 2009 22:25:09 +0200 fixed proof --- fact_setprod removed for fact_altdef_nat
Thu, 23 Jul 2009 21:13:21 +0200 merged
Thu, 23 Jul 2009 21:12:57 +0200 Vandermonde vs Pochhammer; Hypergeometric series - very basic facts
Wed, 15 Jul 2009 06:14:25 +0200 Moved important theorems from FPS_Examples to FPS --- they are not
Fri, 17 Jul 2009 13:12:18 -0400 Changed fact_Suc_nat back to fact_Suc
Tue, 14 Jul 2009 20:58:53 -0400 Repairs regarding new Fact.thy.
Thu, 09 Jul 2009 10:34:51 +0200 FPS form a metric space, which justifies the infinte sum notation
Wed, 24 Jun 2009 09:41:14 +0200 corrected and unified thm names
Tue, 23 Jun 2009 14:24:58 +0200 simplified proof
Tue, 02 Jun 2009 12:18:08 +0200 merged
Mon, 01 Jun 2009 09:26:28 +0200 Reverses idempotent; radical of E; generalized logarithm;
Thu, 28 May 2009 00:49:12 -0700 addition formulas for fps_sin, fps_cos
Thu, 28 May 2009 00:47:17 -0700 use class field_char_0 for fps definitions
Mon, 18 May 2009 23:42:55 +0100 FPS composition distributes over inverses, division and arbitrary nth roots. General geometric series theorem
Thu, 14 May 2009 15:39:15 +0200 Cleaned up Parity a little
Fri, 08 May 2009 19:28:11 +0100 fixed theorem statement
Fri, 08 May 2009 14:02:33 +0100 Generalized distributivity theorems of radicals over multiplication, division and inverses
Wed, 29 Apr 2009 14:20:26 +0200 farewell to class recpower
Sun, 26 Apr 2009 23:40:22 +0100 merged
Fri, 24 Apr 2009 19:29:14 +0100 more general statements
Fri, 24 Apr 2009 17:45:15 +0200 funpow and relpow with shared "^^" syntax
Wed, 22 Apr 2009 19:09:21 +0200 power operation defined generic
Mon, 20 Apr 2009 09:32:07 +0200 power operation on functions with syntax o^; power operation on relations with syntax ^^
Wed, 01 Apr 2009 16:03:00 +0200 added strong_setprod_cong[cong] (in analogy with setsum)