src/HOL/Probability/Sigma_Algebra.thy
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, 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
Tue, 20 May 2014 19:24:39 +0200 hoelzl add various lemmas
Mon, 19 May 2014 13:44:13 +0200 hoelzl fixed document generation for HOL-Probability
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
Tue, 13 May 2014 11:35:47 +0200 hoelzl clean up Lebesgue integration
Sat, 15 Mar 2014 08:31:33 +0100 haftmann more complete set of lemmas wrt. image and composition
Wed, 13 Nov 2013 09:37:00 +0100 hoelzl fix document generation for HOL-Probability
Tue, 12 Nov 2013 19:28:56 +0100 hoelzl measure of a countable union
Tue, 12 Nov 2013 19:28:56 +0100 hoelzl add restrict_space measure
Tue, 24 Sep 2013 10:35:37 +0200 Andreas Lochbihler make measure_of total
Tue, 03 Sep 2013 01:12:40 +0200 wenzelm tuned proofs -- clarified flow of facts wrt. calculation;
Wed, 10 Apr 2013 18:51:21 +0200 hoelzl generalize Borel-set properties from real/ereal/ordered_euclidean_spaces to order_topology and real_normed_vector
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
Wed, 05 Dec 2012 15:59:08 +0100 hoelzl Move the measurability prover to its own file
Wed, 05 Dec 2012 15:58:48 +0100 hoelzl Show search depth in the debug output of the measurability prover
Thu, 29 Nov 2012 09:59:20 +0100 hoelzl make SML/NJ happy (give names for all fields in a record)
Wed, 28 Nov 2012 15:59:18 +0100 wenzelm eliminated slightly odd identifiers;
Tue, 27 Nov 2012 13:48:40 +0100 immler based countable topological basis on Countable_Set
Tue, 27 Nov 2012 11:29:47 +0100 immler qualified interpretation of sigma_algebra, to avoid name clashes
Fri, 16 Nov 2012 12:10:02 +0100 hoelzl more measurability rules
Tue, 06 Nov 2012 19:18:35 +0100 hoelzl add support for function application to measurability prover
Fri, 02 Nov 2012 14:23:54 +0100 hoelzl use measurability prover
Fri, 02 Nov 2012 14:23:40 +0100 hoelzl add measurability prover; add support for Borel sets
Fri, 12 Oct 2012 18:58:20 +0200 wenzelm discontinued obsolete typedef (open) syntax;
Wed, 10 Oct 2012 12:12:27 +0200 hoelzl add induction rule for intersection-stable sigma-sets
Wed, 10 Oct 2012 12:12:22 +0200 hoelzl add measurable_compose
Wed, 10 Oct 2012 12:12:15 +0200 hoelzl tuned measurable_If; moved countably_additive equalities to Measure_Space; tuned proofs
Wed, 25 Apr 2012 19:26:27 +0200 hoelzl add Caratheodories theorem for semi-rings of sets
Wed, 25 Apr 2012 15:06:59 +0200 hoelzl correct lemma name
Mon, 23 Apr 2012 12:14:35 +0200 hoelzl reworked Probability theory
Tue, 28 Feb 2012 21:53:36 +0100 wenzelm avoid undeclared variables in let bindings;
Mon, 12 Sep 2011 07:55:43 +0200 nipkow new fastforce replacing fastsimp - less confusing name
Fri, 26 Aug 2011 15:00:00 -0700 huffman make HOL-Probability respect set/pred distinction
Tue, 09 Aug 2011 20:24:48 +0200 haftmann tuned proofs
Thu, 26 May 2011 17:40:01 +0200 hoelzl add lemma indep_distribution_eq_measure
Thu, 26 May 2011 14:12:06 +0200 hoelzl add lemma indep_rv_finite
Thu, 26 May 2011 14:12:01 +0200 hoelzl add lemma sigma_sets_singleton
Thu, 26 May 2011 14:11:57 +0200 hoelzl add lemma indep_sets_collect_sigma
Tue, 17 May 2011 15:00:39 +0200 hoelzl Collect intro-rules for sigma-algebras
Tue, 17 May 2011 12:22:58 +0200 hoelzl add measurable_Least
Tue, 17 May 2011 12:22:40 +0200 hoelzl add restrict_sigma
Tue, 29 Mar 2011 14:27:31 +0200 hoelzl proved caratheodory_empty_continuous
Tue, 22 Mar 2011 20:06:10 +0100 hoelzl standardized headers
Tue, 22 Mar 2011 16:44:57 +0100 hoelzl add ring_of_sets and subset_class as basis for algebra
Mon, 14 Mar 2011 16:59:37 +0100 wenzelm standardized headers;
Mon, 14 Mar 2011 14:37:49 +0100 hoelzl reworked Probability theory: measures are not type restricted to positive extended reals
Sun, 13 Mar 2011 22:55:50 +0100 wenzelm tuned headers;
Fri, 04 Feb 2011 14:16:48 +0100 hoelzl add borel_fubini_integrable; remove unused bijectivity rules for measureable functions
Wed, 02 Feb 2011 12:34:45 +0100 hoelzl the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
Fri, 14 Jan 2011 14:21:26 +0100 hoelzl tuned theorem order
Wed, 29 Dec 2010 17:34:41 +0100 wenzelm explicit file specifications -- avoid secondary load path;
Wed, 08 Dec 2010 16:15:14 +0100 hoelzl cleanup bijectivity btw. product spaces and pairs
Wed, 01 Dec 2010 21:03:02 +0100 hoelzl Generalized simple_functionD and less_SUP_iff.
Wed, 01 Dec 2010 20:09:41 +0100 hoelzl Replace algebra_eqI by algebra.equality;
Wed, 01 Dec 2010 19:20:30 +0100 hoelzl Support product spaces on sigma finite measures.
Mon, 22 Nov 2010 10:34:33 +0100 hoelzl Replace surj by abbreviation; remove surj_on.
Wed, 06 Oct 2010 17:38:06 +0200 blanchet remove needless fact
less more (0) -60 tip