src/HOL/Limits.thy
Thu, 29 Oct 2015 15:40:52 +0100 eberlm added many small lemmas about setsum/setprod/powr/...
Sun, 13 Sep 2015 22:56:52 +0200 wenzelm tuned proofs -- less legacy;
Tue, 01 Sep 2015 22:32:58 +0200 wenzelm eliminated \<Colon>;
Wed, 19 Aug 2015 19:18:19 +0100 paulson New material and fixes related to the forthcoming Stone-Weierstrass development
Sat, 18 Jul 2015 22:58:50 +0200 wenzelm isabelle update_cartouches;
Tue, 14 Jul 2015 13:48:03 +0200 hoelzl generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
Thu, 07 May 2015 15:34:28 +0200 hoelzl generalized tends over powr; added DERIV rule for powr
Tue, 21 Apr 2015 17:19:00 +0100 paulson New material, mostly about limits. Consolidation.
Sat, 11 Apr 2015 11:56:40 +0100 paulson Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
Tue, 31 Mar 2015 21:54:32 +0200 haftmann given up separate type classes demanding `inverse 0 = 0`
Thu, 05 Mar 2015 17:30:29 +0000 paulson The function frac. Various lemmas about limits, series, the exp function, etc.
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Mon, 20 Oct 2014 18:33:14 +0200 hoelzl add tendsto_const and tendsto_ident_at as simp and intro rules
Fri, 04 Jul 2014 20:18:47 +0200 haftmann reduced name variants for assoc and commute on plus and mult
Mon, 30 Jun 2014 15:45:21 +0200 hoelzl import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
Wed, 18 Jun 2014 14:31:32 +0200 hoelzl filters are easier to define with INF on filters.
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, 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, 02 Apr 2014 18:35:07 +0200 hoelzl extend continuous_intros; remove continuous_on_intros and isCont_intros
Wed, 02 Apr 2014 16:45:31 +0100 paulson new theorem about zero limits
Mon, 31 Mar 2014 12:16:39 +0200 hoelzl add limits of power at top and bot
Wed, 12 Feb 2014 08:35:57 +0100 blanchet renamed 'nat_{case,rec}' to '{case,rec}_nat'
Wed, 25 Dec 2013 17:39:06 +0100 haftmann prefer more canonical names for lemmas on min/max
Tue, 05 Nov 2013 09:45:02 +0100 hoelzl move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
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
Tue, 03 Sep 2013 22:04:23 +0200 wenzelm tuned proofs -- less guessing;
Thu, 30 May 2013 23:29:33 +0200 wenzelm tuned headers;
Tue, 09 Apr 2013 14:04:47 +0200 hoelzl move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
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)
Tue, 26 Mar 2013 12:21:01 +0100 hoelzl remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
Tue, 26 Mar 2013 12:21:00 +0100 hoelzl move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
Tue, 26 Mar 2013 12:20:58 +0100 hoelzl move SEQ.thy and Lim.thy to Limits.thy
Tue, 26 Mar 2013 12:20:57 +0100 hoelzl rename RealVector.thy to Real_Vector_Spaces.thy
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)
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
Fri, 22 Mar 2013 10:41:43 +0100 hoelzl move metric_space to its own theory
Fri, 22 Mar 2013 10:41:42 +0100 hoelzl move topological_space to its own theory
Wed, 06 Mar 2013 16:56:21 +0100 hoelzl add tendsto_eq_intros: they add an additional rewriting step at the rhs of --->
Wed, 20 Feb 2013 12:04:42 +0100 hoelzl move auxiliary lemmas from Library/Extended_Reals to HOL image
Wed, 06 Feb 2013 17:57:21 +0100 hoelzl replace open_interval with the rule open_tendstoI; generalize Liminf/Limsup rules
Thu, 31 Jan 2013 11:31:27 +0100 hoelzl introduce order topology
Mon, 14 Jan 2013 17:16:59 +0100 hoelzl move eventually_Ball_finite to Limits
Fri, 07 Dec 2012 14:29:09 +0100 hoelzl add exponential and uniform distributions
Tue, 04 Dec 2012 18:00:37 +0100 hoelzl prove tendsto_power_div_exp_0
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
Mon, 03 Dec 2012 18:19:12 +0100 hoelzl use filterlim in Lim and SEQ; tuned proofs
Mon, 03 Dec 2012 18:19:11 +0100 hoelzl conversion rules for at, at_left and at_right; applied to l'Hopital's rules.
Mon, 03 Dec 2012 18:19:07 +0100 hoelzl add L'Hôpital's rule
Mon, 03 Dec 2012 18:19:05 +0100 hoelzl add filterlim rules for exp and ln to infinity
Mon, 03 Dec 2012 18:19:04 +0100 hoelzl add filterlim rules for inverse and at_infinity
Mon, 03 Dec 2012 18:19:02 +0100 hoelzl add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
Mon, 03 Dec 2012 18:19:01 +0100 hoelzl add filterlim rules for unary minus and inverse
Mon, 03 Dec 2012 18:18:59 +0100 hoelzl rename filter_lim to filterlim to be consistent with filtermap
Tue, 27 Nov 2012 19:31:11 +0100 hoelzl introduce filter_lim as a generatlization of tendsto
Fri, 12 Oct 2012 18:58:20 +0200 wenzelm discontinued obsolete typedef (open) syntax;
Thu, 12 Apr 2012 18:39:19 +0200 wenzelm more standard method setup;
Mon, 12 Mar 2012 21:34:43 +0100 noschinl use eventually_elim method
Mon, 12 Mar 2012 21:28:10 +0100 noschinl add eventually_elim method
less more (0) -100 -60 tip