src/HOL/Library/Float.thy
Tue, 21 Feb 2012 16:28:18 +0100 misc tuning;
Thu, 29 Dec 2011 10:47:55 +0100 attribute code_abbrev superseedes code_unfold_post
Tue, 06 Dec 2011 14:29:37 +0100 tuned proofs
Mon, 14 Nov 2011 18:36:31 +0100 cleaned up float theories; removed duplicate definitions and theorems
Tue, 06 Sep 2011 19:03:41 -0700 avoid using legacy theorem names
Wed, 04 May 2011 15:37:39 +0200 proper case_names for int_cases, int_of_nat_induct;
Wed, 12 Jan 2011 17:14:27 +0100 eliminated global prems;
Mon, 06 Dec 2010 19:54:48 +0100 move coercions to appropriate places
Mon, 06 Sep 2010 15:01:37 +0200 When comparing Floats use integers instead of reals (represented as rationals), generates less code when Floats are used.
Sun, 09 May 2010 22:51:11 -0700 avoid using real-specific versions of generic lemmas
Tue, 23 Feb 2010 10:37:25 -0800 moved some lemmas from RealPow to RealDef; changed orientation of real_of_int_power
Mon, 08 Feb 2010 14:06:41 +0100 separate library theory for type classes combining lattices with various algebraic structures
Tue, 10 Nov 2009 18:29:07 +0100 eliminated some old uses of cumulative prems (!) in proof methods;
Sat, 17 Oct 2009 14:43:18 +0200 eliminated hard tabulators, guessing at each author's individual tab-width;
Tue, 14 Jul 2009 16:27:32 +0200 prefer code_inline over code_unfold; use code_unfold_post where appropriate
Tue, 14 Jul 2009 10:54:04 +0200 code attributes use common underscore convention
Mon, 29 Jun 2009 23:29:11 +0200 Implemented taylor series expansion for approximation
Thu, 04 Jun 2009 17:55:47 +0200 Approximation: Implemented argument reduction for cosine. Sinus is now implemented in terms of cosine. Sqrt computes on the entire real numbers
Wed, 29 Apr 2009 20:19:50 +0200 replaced Ifloat => real_of_float and real, renamed ApproxEq => inequality, uneq => interpret_inequality, uneq' => approx_inequality, Ifloatarith => interpret_floatarith
Wed, 29 Apr 2009 14:20:26 +0200 farewell to class recpower
Wed, 22 Apr 2009 19:09:21 +0200 power operation defined generic
Wed, 04 Mar 2009 11:05:29 +0100 Merge.
Wed, 04 Mar 2009 10:45:52 +0100 Merge.
Sun, 01 Mar 2009 12:01:57 +0100 removed redundant lemmas
Thu, 26 Feb 2009 20:56:59 +0100 standard headers;
Sat, 21 Feb 2009 09:58:26 +0100 removed redundant thms
Wed, 18 Feb 2009 20:53:58 -0800 add header
Thu, 05 Feb 2009 11:45:15 +0100 Added new Float theory and moved old Library/Float.thy to ComputeFloat
Wed, 28 Jan 2009 16:29:16 +0100 Replaced group_ and ring_simps by algebra_simps;
Tue, 09 Dec 2008 22:13:16 -0800 move all neg-related lemmas to NatBin; make type of neg specific to int
Wed, 03 Dec 2008 21:50:36 -0800 enable eq_bin_simps for simplifying equalities on numerals
Wed, 03 Dec 2008 21:00:39 -0800 fix proofs related to simplification of inequalities on numerals
Wed, 03 Dec 2008 15:58:44 +0100 made repository layout more coherent with logical distribution structure; stripped some $Id$s