src/HOL/Transcendental.thy
Thu, 19 Mar 2015 14:24:51 +0000 paulson New material for complex sin, cos, tan, Ln, also some reorganisation
Wed, 18 Mar 2015 17:23:22 +0000 paulson new HOL Light material about exp, sin, cos
Wed, 18 Mar 2015 14:13:27 +0000 paulson Lots of new material on complex-valued functions. Modified simplification of (x/n)^k
Tue, 17 Mar 2015 12:23:56 +0000 paulson Merge
Mon, 16 Mar 2015 15:30:00 +0000 paulson The factorial function, "fact", now has type "nat => 'a"
Fri, 13 Mar 2015 12:44:16 +0100 wenzelm removed junk;
Tue, 10 Mar 2015 16:12:35 +0000 paulson renaming HOL/Fact.thy -> Binomial.thy
Mon, 09 Mar 2015 16:28:19 +0000 paulson sin, cos generalised from type real to any "'a::{real_normed_field,banach}", including complex
Sat, 07 Mar 2015 21:32:31 +0100 wenzelm clarified Drule.gen_all: observe context more carefully;
Thu, 05 Mar 2015 17:30:29 +0000 paulson The function frac. Various lemmas about limits, series, the exp function, etc.
Wed, 04 Mar 2015 23:31:04 +0100 nipkow Removed the obsolete functions "natfloor" and "natceiling"
Wed, 12 Nov 2014 17:36:36 +0100 immler added lemmas: convert between powr and log in comparisons, pull log out of addition/subtraction
Wed, 12 Nov 2014 17:36:25 +0100 immler code equation for powr
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
Tue, 21 Oct 2014 21:10:44 +0200 haftmann turn even into an abbreviation
Mon, 20 Oct 2014 18:33:14 +0200 hoelzl add tendsto_const and tendsto_ident_at as simp and intro rules
Mon, 20 Oct 2014 07:45:58 +0200 haftmann augmented and tuned facts on even/odd and division
Sun, 19 Oct 2014 18:05:26 +0200 haftmann prefer generic elimination rules for even/odd over specialized unfold rules for nat
Mon, 13 Oct 2014 18:55:05 +0200 immler relaxed class constraints for exp
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
Sat, 28 Jun 2014 09:16:42 +0200 haftmann fact consolidation
Wed, 18 Jun 2014 07:31:12 +0200 hoelzl moved lemmas from the proof of the Central Limit Theorem by Jeremy Avigad and Luke Serafin
Fri, 06 Jun 2014 12:36:06 +0200 nipkow added lemma
Fri, 30 May 2014 14:55:10 +0200 hoelzl introduce more powerful reindexing rules for big operators
Tue, 20 May 2014 19:24:39 +0200 hoelzl add various lemmas
Tue, 13 May 2014 22:14:12 +0200 nipkow added lemmas
Mon, 14 Apr 2014 13:08:17 +0200 hoelzl added divide_nonneg_nonneg and co; made it a simp rule
Sat, 12 Apr 2014 17:26:27 +0200 nipkow made mult_pos_pos a simp rule
Fri, 11 Apr 2014 22:53:33 +0200 nipkow made divide_pos_pos a simp rule
Fri, 11 Apr 2014 13:36:57 +0200 nipkow made mult_nonneg_nonneg a simp rule
Wed, 09 Apr 2014 13:15:21 +0200 hoelzl generalize ln/log_powr; add log_base_powr/pow
Wed, 09 Apr 2014 09:37:47 +0200 hoelzl revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules
Thu, 03 Apr 2014 23:51:52 +0100 paulson removing simprule status for divide_minus_left and divide_minus_right
Thu, 03 Apr 2014 17:56:08 +0200 hoelzl merged DERIV_intros, has_derivative_intros into derivative_intros
Wed, 02 Apr 2014 18:35:07 +0200 hoelzl extend continuous_intros; remove continuous_on_intros and isCont_intros
Mon, 24 Mar 2014 14:22:29 +0000 paulson rearranging some deriv theorems
Wed, 19 Mar 2014 17:06:02 +0000 paulson Some rationalisation of basic lemmas
Wed, 19 Mar 2014 15:34:57 +0100 hoelzl further renaming in Series
Tue, 18 Mar 2014 15:53:48 +0100 hoelzl cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
Mon, 17 Mar 2014 19:12:52 +0100 hoelzl unify syntax for has_derivative and differentiable
Sun, 16 Mar 2014 13:34:35 -0700 huffman tuned proofs
Sun, 02 Mar 2014 18:11:30 +0100 wenzelm repaired document;
Tue, 25 Feb 2014 16:17:20 +0000 paulson More complex-related lemmas
Mon, 24 Feb 2014 16:56:04 +0000 paulson Lemmas about Reals, norm, etc., and cleaner variants of existing ones
Wed, 12 Feb 2014 08:37:06 +0100 blanchet adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
Mon, 25 Nov 2013 00:02:39 +0000 paulson tidied more proofs
Sun, 24 Nov 2013 18:37:25 +0000 paulson cleaned up more messy proofs
Sun, 24 Nov 2013 13:06:22 +0000 paulson cleaned up some messy proofs
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
Fri, 13 Sep 2013 07:59:50 +0200 haftmann tuned proofs
Thu, 12 Sep 2013 15:08:46 -0700 huffman generalize lemmas
Sun, 18 Aug 2013 22:44:39 +0200 wenzelm tuned proofs;
Sun, 18 Aug 2013 18:49:45 +0200 wenzelm more symbols;
Tue, 13 Aug 2013 16:25:47 +0200 wenzelm standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
Sat, 25 May 2013 13:59:08 +0200 noschinl add lemma
less more (0) -100 -60 tip