src/HOL/Probability/Lebesgue_Measure.thy
Fri, 29 Jul 2016 20:34:07 +0200 wenzelm more accurate cong del;
Fri, 22 Jul 2016 11:00:43 +0200 wenzelm tuned proofs -- avoid unstructured calculation;
Thu, 09 Jun 2016 16:11:33 +0200 hoelzl remove smt call in Lebesge_Measure
Mon, 25 Apr 2016 16:09:26 +0200 wenzelm eliminated old 'def';
Thu, 14 Apr 2016 15:48:11 +0200 hoelzl Probability: move emeasure and nn_integral from ereal to ennreal
Tue, 23 Feb 2016 16:25:08 +0100 nipkow more canonical names
Wed, 17 Feb 2016 21:51:56 +0100 haftmann prefer abbreviations for compound operators INFIMUM and SUPREMUM
Wed, 30 Dec 2015 11:21:54 +0100 wenzelm more symbols;
Tue, 29 Dec 2015 23:04:53 +0100 wenzelm more symbols;
Mon, 28 Dec 2015 19:23:15 +0100 wenzelm more symbols;
Mon, 28 Dec 2015 01:28:28 +0100 wenzelm more symbols;
Mon, 07 Dec 2015 20:19:59 +0100 wenzelm isabelle update_cartouches -c -t;
Tue, 01 Dec 2015 14:09:10 +0000 paulson Removal of redundant lemmas (diff_less_iff, diff_le_iff) and of the abbreviation Exp. Addition of some new material.
Tue, 10 Nov 2015 14:43:29 +0000 paulson Merge
Tue, 10 Nov 2015 14:18:41 +0000 paulson Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
Mon, 09 Nov 2015 15:48:17 +0100 wenzelm qualifier is mandatory by default;
Wed, 30 Sep 2015 16:36:42 +0100 paulson real_of_nat_Suc is now a simprule
Tue, 30 Jun 2015 13:56:16 +0100 paulson Useful lemmas. The theorem concerning swapping the variables in a double integral.
Wed, 18 Mar 2015 14:13:27 +0000 paulson Lots of new material on complex-valued functions. Modified simplification of (x/n)^k
Wed, 18 Feb 2015 22:46:47 +0100 haftmann inlined rules to free user-space from technical names
Thu, 22 Jan 2015 14:51:08 +0100 hoelzl import general thms from Density_Compiler
Wed, 14 Jan 2015 10:15:41 +0100 Andreas Lochbihler allow line breaks in integral notation
Mon, 24 Nov 2014 12:20:14 +0100 hoelzl add congruence solver to measurability prover
Thu, 13 Nov 2014 17:19:52 +0100 hoelzl import general theorems from AFP/Markov_Models
Sun, 02 Nov 2014 17:06:05 +0100 wenzelm modernized header;
Sun, 26 Oct 2014 19:11:16 +0100 haftmann eliminated redundancies;
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
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 07:31:12 +0200 hoelzl moved lemmas from the proof of the Central Limit Theorem by Jeremy Avigad and Luke Serafin
Thu, 12 Jun 2014 15:47:36 +0200 hoelzl properties of Erlang and exponentially distributed random variables (by Sudeep Kanav)
Tue, 03 Jun 2014 16:22:01 +0200 hoelzl use 0 as integral-value for non-integrable functions, simplify a couple of rewrite rules
Fri, 30 May 2014 18:48:05 +0200 hoelzl generalizd measurability on restricted space; rule for integrability on compact sets
Fri, 30 May 2014 15:56:30 +0200 hoelzl better support for restrict_space
Mon, 19 May 2014 14:26:58 +0200 hoelzl renamed positive_integral to nn_integral
Mon, 19 May 2014 12:04:45 +0200 hoelzl introduce Bochner integral: generalizes Lebesgue integral from real-valued function to functions on real-normed vector spaces
Wed, 19 Mar 2014 18:47:22 +0100 haftmann elongated INFI and SUPR, to reduced risk of confusing theorems names in the future while still being consistent with INTER and UNION
Tue, 18 Mar 2014 15:53:48 +0100 hoelzl cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
Tue, 18 Mar 2014 10:12:57 +0100 immler use cbox to relax class constraints
Mon, 17 Mar 2014 19:12:52 +0100 hoelzl unify syntax for has_derivative and differentiable
Mon, 10 Mar 2014 20:04:40 +0100 hoelzl introduced antimono; incseq, decseq are now abbreviations for mono and antimono; renamed Library/Continuity to Library/Order_Continuity; removed up_cont; renamed down_cont to down_continuity and generalized to complete_lattices
Wed, 25 Dec 2013 17:39:06 +0100 haftmann prefer more canonical names for lemmas on min/max
Mon, 16 Dec 2013 17:08:22 +0100 immler prefer box over greaterThanLessThan on euclidean_space
Tue, 05 Nov 2013 09:44:57 +0100 hoelzl generalize SUP and INF to the syntactic type classes Sup and Inf
Tue, 03 Sep 2013 01:12:40 +0200 wenzelm tuned proofs -- clarified flow of facts wrt. calculation;
Tue, 13 Aug 2013 16:25:47 +0200 wenzelm standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
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)
Thu, 31 Jan 2013 11:31:30 +0100 hoelzl use order topology for extended reals
Fri, 14 Dec 2012 15:46:01 +0100 hoelzl Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
Fri, 07 Dec 2012 14:29:08 +0100 hoelzl fundamental theorem of calculus for the Lebesgue integral
Wed, 05 Dec 2012 15:58:45 +0100 hoelzl Remove looping rule from measurability prover
Tue, 27 Nov 2012 11:29:47 +0100 immler qualified interpretation of sigma_algebra, to avoid name clashes
Mon, 19 Nov 2012 12:29:02 +0100 hoelzl merge extensional dependent function space from FuncSet with the one in Finite_Product_Measure
Fri, 16 Nov 2012 19:14:23 +0100 hoelzl moved (b)choice_iff(') to Hilbert_Choice
Fri, 16 Nov 2012 18:45:57 +0100 hoelzl move theorems to be more generally useable
Fri, 02 Nov 2012 14:23:54 +0100 hoelzl use measurability prover
Wed, 10 Oct 2012 12:12:35 +0200 hoelzl add induction for real Borel measurable functions
Wed, 10 Oct 2012 12:12:23 +0200 hoelzl remove incseq assumption from measure_eqI_generator_eq
Wed, 10 Oct 2012 12:12:20 +0200 hoelzl remove incseq assumption from sigma_prod_algebra_sigma_eq
Wed, 10 Oct 2012 12:12:18 +0200 hoelzl tuned Lebesgue measure proofs
less more (0) -60 tip