| Sun, 18 Aug 2013 22:44:39 +0200 | 
wenzelm | 
tuned proofs;
 | 
file |
diff |
annotate
 | 
| Sun, 18 Aug 2013 18:49:45 +0200 | 
wenzelm | 
more symbols;
 | 
file |
diff |
annotate
 | 
| Tue, 13 Aug 2013 16:25:47 +0200 | 
wenzelm | 
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 | 
file |
diff |
annotate
 | 
| Sat, 25 May 2013 13:59:08 +0200 | 
noschinl | 
add lemma
 | 
file |
diff |
annotate
 | 
| Tue, 09 Apr 2013 14:04:41 +0200 | 
hoelzl | 
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 | 
file |
diff |
annotate
 | 
| Tue, 26 Mar 2013 12:20:59 +0100 | 
hoelzl | 
move Ln.thy and Log.thy to Transcendental.thy
 | 
file |
diff |
annotate
 | 
| Fri, 22 Mar 2013 10:41:43 +0100 | 
hoelzl | 
arcsin and arccos are continuous on {0 .. 1} (including the endpoints)
 | 
file |
diff |
annotate
 | 
| Fri, 22 Mar 2013 10:41:43 +0100 | 
hoelzl | 
move continuous_on_inv to HOL image (simplifies isCont_inverse_function)
 | 
file |
diff |
annotate
 | 
| Fri, 22 Mar 2013 10:41:43 +0100 | 
hoelzl | 
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 | 
file |
diff |
annotate
 | 
| Fri, 22 Mar 2013 10:41:43 +0100 | 
hoelzl | 
clean up lemma_nest_unique and renamed to nested_sequence_unique
 | 
file |
diff |
annotate
 | 
| Tue, 04 Dec 2012 18:00:37 +0100 | 
hoelzl | 
prove tendsto_power_div_exp_0
 | 
file |
diff |
annotate
 | 
| Tue, 04 Dec 2012 18:00:31 +0100 | 
hoelzl | 
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 | 
file |
diff |
annotate
 | 
| Mon, 03 Dec 2012 18:19:05 +0100 | 
hoelzl | 
add filterlim rules for exp and ln to infinity
 | 
file |
diff |
annotate
 | 
| Fri, 19 Oct 2012 15:12:52 +0200 | 
webertj | 
Renamed {left,right}_distrib to distrib_{right,left}.
 | 
file |
diff |
annotate
 | 
| Mon, 16 Apr 2012 11:24:57 +0200 | 
huffman | 
tuned some proofs;
 | 
file |
diff |
annotate
 | 
| Sun, 25 Mar 2012 20:15:39 +0200 | 
huffman | 
merged fork with new numeral representation (see NEWS)
 | 
file |
diff |
annotate
 | 
| Tue, 17 Jan 2012 16:30:54 +0100 | 
huffman | 
factor-cancellation simprocs now call the full simplifier to prove that factors are non-zero
 | 
file |
diff |
annotate
 | 
| Thu, 15 Dec 2011 17:21:29 +0100 | 
huffman | 
tendsto lemmas for ln and powr
 | 
file |
diff |
annotate
 | 
| Sun, 30 Oct 2011 09:42:13 +0100 | 
huffman | 
removed ad-hoc simp rules sin_cos_eq[symmetric], minus_sin_cos_eq[symmetric], cos_sin_eq[symmetric]
 | 
file |
diff |
annotate
 | 
| Sun, 30 Oct 2011 09:07:02 +0100 | 
huffman | 
extend cancellation simproc patterns to cover terms like '- (2 * pi) < pi'
 | 
file |
diff |
annotate
 | 
| Tue, 06 Sep 2011 10:30:00 -0700 | 
huffman | 
simplify proof of tan_half, removing unused assumptions
 | 
file |
diff |
annotate
 | 
| Tue, 06 Sep 2011 09:56:09 -0700 | 
huffman | 
convert some proofs to Isar-style
 | 
file |
diff |
annotate
 | 
| Mon, 05 Sep 2011 22:30:25 -0700 | 
huffman | 
add lemmas about arctan;
 | 
file |
diff |
annotate
 | 
| Mon, 05 Sep 2011 18:06:02 -0700 | 
huffman | 
convert lemma cos_total to Isar-style proof
 | 
file |
diff |
annotate
 | 
| Mon, 05 Sep 2011 17:45:37 -0700 | 
huffman | 
convert lemma cos_is_zero to Isar-style
 | 
file |
diff |
annotate
 | 
| Mon, 05 Sep 2011 17:00:56 -0700 | 
huffman | 
convert lemma sin_gt_zero to Isar style;
 | 
file |
diff |
annotate
 | 
| Mon, 05 Sep 2011 16:26:57 -0700 | 
huffman | 
modify lemma sums_group, and shorten proofs that use it
 | 
file |
diff |
annotate
 | 
| Mon, 05 Sep 2011 16:07:40 -0700 | 
huffman | 
generalize some lemmas
 | 
file |
diff |
annotate
 | 
| Mon, 05 Sep 2011 12:19:04 -0700 | 
huffman | 
add lemmas cos_arctan and sin_arctan
 | 
file |
diff |
annotate
 | 
| Sun, 04 Sep 2011 09:49:45 -0700 | 
huffman | 
remove redundant lemmas about LIMSEQ
 | 
file |
diff |
annotate
 | 
| Sun, 28 Aug 2011 09:20:12 -0700 | 
huffman | 
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 | 
file |
diff |
annotate
 | 
| Fri, 19 Aug 2011 18:42:41 -0700 | 
huffman | 
move sin_coeff and cos_coeff lemmas to Transcendental.thy; simplify some proofs
 | 
file |
diff |
annotate
 | 
| Fri, 19 Aug 2011 18:08:05 -0700 | 
huffman | 
remove unused lemma DERIV_sin_add
 | 
file |
diff |
annotate
 | 
| Fri, 19 Aug 2011 18:06:27 -0700 | 
huffman | 
remove redundant lemma lemma_DERIV_subst in favor of DERIV_cong
 | 
file |
diff |
annotate
 | 
| Fri, 19 Aug 2011 17:59:19 -0700 | 
huffman | 
remove redundant lemma exp_ln_eq in favor of ln_unique
 | 
file |
diff |
annotate
 | 
| Fri, 19 Aug 2011 14:17:28 -0700 | 
huffman | 
Transcendental.thy: add tendsto_intros lemmas;
 | 
file |
diff |
annotate
 | 
| Fri, 19 Aug 2011 10:46:54 -0700 | 
huffman | 
Transcendental.thy: remove several unused lemmas and simplify some proofs
 | 
file |
diff |
annotate
 | 
| Fri, 19 Aug 2011 08:40:15 -0700 | 
huffman | 
remove unused lemmas
 | 
file |
diff |
annotate
 | 
| Fri, 19 Aug 2011 07:45:22 -0700 | 
huffman | 
remove some redundant simp rules
 | 
file |
diff |
annotate
 | 
| Thu, 18 Aug 2011 19:53:03 -0700 | 
huffman | 
optimize some proofs
 | 
file |
diff |
annotate
 | 
| Thu, 18 Aug 2011 13:36:58 -0700 | 
huffman | 
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 | 
file |
diff |
annotate
 | 
| Tue, 31 May 2011 21:33:49 +0200 | 
hoelzl | 
use divide instead of inverse for the derivative of ln
 | 
file |
diff |
annotate
 | 
| Mon, 14 Mar 2011 14:37:35 +0100 | 
hoelzl | 
generalize infinite sums
 | 
file |
diff |
annotate
 | 
| Fri, 14 Jan 2011 15:44:47 +0100 | 
wenzelm | 
eliminated global prems;
 | 
file |
diff |
annotate
 | 
| Mon, 23 Aug 2010 11:17:13 +0200 | 
haftmann | 
dropped type classes mult_mono and mult_mono1; tuned names of technical rule duplicates
 | 
file |
diff |
annotate
 | 
| Mon, 19 Jul 2010 16:09:44 +0200 | 
haftmann | 
diff_minus subsumes diff_def
 | 
file |
diff |
annotate
 | 
| Mon, 17 May 2010 15:58:32 -0700 | 
huffman | 
remove some unnamed simp rules from Transcendental.thy; move the needed ones to MacLaurin.thy where they are used
 | 
file |
diff |
annotate
 | 
| Mon, 17 May 2010 08:45:46 -0700 | 
huffman | 
remove simp attribute from square_eq_1_iff
 | 
file |
diff |
annotate
 | 
| Tue, 11 May 2010 19:38:16 -0700 | 
huffman | 
fix some linarith_split_limit warnings
 | 
file |
diff |
annotate
 | 
| Tue, 11 May 2010 06:30:48 -0700 | 
huffman | 
move some theorems from RealPow.thy to Transcendental.thy
 | 
file |
diff |
annotate
 | 
| Sun, 09 May 2010 17:47:43 -0700 | 
huffman | 
avoid using real-specific versions of generic lemmas
 | 
file |
diff |
annotate
 | 
| Sun, 09 May 2010 14:21:44 -0700 | 
huffman | 
remove a couple of redundant lemmas; simplify some proofs
 | 
file |
diff |
annotate
 | 
| Thu, 18 Feb 2010 14:21:44 -0800 | 
huffman | 
get rid of many duplicate simp rule warnings
 | 
file |
diff |
annotate
 | 
| Thu, 18 Feb 2010 08:08:51 -0800 | 
huffman | 
fix looping call to simplifier
 | 
file |
diff |
annotate
 | 
| Mon, 08 Feb 2010 14:06:58 +0100 | 
haftmann | 
more precise proofs
 | 
file |
diff |
annotate
 | 
| Fri, 05 Feb 2010 14:33:50 +0100 | 
haftmann | 
more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
 | 
file |
diff |
annotate
 | 
| Thu, 28 Jan 2010 11:48:49 +0100 | 
haftmann | 
new theory Algebras.thy for generic algebraic structures
 | 
file |
diff |
annotate
 | 
| Fri, 13 Nov 2009 17:15:12 +0000 | 
paulson | 
A little rationalisation
 | 
file |
diff |
annotate
 | 
| Tue, 10 Nov 2009 14:38:06 +0100 | 
wenzelm | 
tuned proofs;
 | 
file |
diff |
annotate
 | 
| Sat, 17 Oct 2009 14:43:18 +0200 | 
wenzelm | 
eliminated hard tabulators, guessing at each author's individual tab-width;
 | 
file |
diff |
annotate
 |