History log of /seL4-l4v-master/isabelle/src/HOL/Probability/Information.thy
Revision Date Author Comments
# 504acaca 14-Jan-2019 haftmann <none@none>

tuned proofs


# 6effda26 14-Jan-2019 nipkow <none@none>

uniform naming


# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# 6fd6219b 21-Oct-2018 nipkow <none@none>

uniform naming of strong congruence rules


# 6e0cccd7 15-Apr-2018 paulson <lp15@cam.ac.uk>

various new results on measures, integrals, etc., and some simplified proofs


# 351cc2e6 17-Oct-2016 nipkow <none@none>

setsum -> sum


# fad39d02 30-Sep-2016 hoelzl <none@none>

HOL-Probability: more about probability, prepare for Markov processes in the AFP

--HG--
extra : rebase_source : f90e6cf5c47f7a2604d0eeacaf0181f3cfe64a14


# 78a9e4a8 16-Sep-2016 hoelzl <none@none>

move Henstock-Kurzweil integration after Lebesgue_Measure; replace content by abbreviation measure lborel

--HG--
extra : rebase_source : 0321297c249a436ca0371010a76a1a026dd33222


# 9e5f909f 05-Aug-2016 hoelzl <none@none>

move measure theory from HOL-Probability to HOL-Multivariate_Analysis

--HG--
rename : src/HOL/Probability/Binary_Product_Measure.thy => src/HOL/Multivariate_Analysis/Binary_Product_Measure.thy
rename : src/HOL/Probability/Bochner_Integration.thy => src/HOL/Multivariate_Analysis/Bochner_Integration.thy
rename : src/HOL/Probability/Borel_Space.thy => src/HOL/Multivariate_Analysis/Borel_Space.thy
rename : src/HOL/Probability/Caratheodory.thy => src/HOL/Multivariate_Analysis/Caratheodory.thy
rename : src/HOL/Probability/Complete_Measure.thy => src/HOL/Multivariate_Analysis/Complete_Measure.thy
rename : src/HOL/Probability/Embed_Measure.thy => src/HOL/Multivariate_Analysis/Embed_Measure.thy
rename : src/HOL/Probability/Finite_Product_Measure.thy => src/HOL/Multivariate_Analysis/Finite_Product_Measure.thy
rename : src/HOL/Probability/Interval_Integral.thy => src/HOL/Multivariate_Analysis/Interval_Integral.thy
rename : src/HOL/Probability/Lebesgue_Integral_Substitution.thy => src/HOL/Multivariate_Analysis/Lebesgue_Integral_Substitution.thy
rename : src/HOL/Probability/Lebesgue_Measure.thy => src/HOL/Multivariate_Analysis/Lebesgue_Measure.thy
rename : src/HOL/Probability/Measurable.thy => src/HOL/Multivariate_Analysis/Measurable.thy
rename : src/HOL/Probability/Measure_Space.thy => src/HOL/Multivariate_Analysis/Measure_Space.thy
rename : src/HOL/Probability/Nonnegative_Lebesgue_Integration.thy => src/HOL/Multivariate_Analysis/Nonnegative_Lebesgue_Integration.thy
rename : src/HOL/Probability/Radon_Nikodym.thy => src/HOL/Multivariate_Analysis/Radon_Nikodym.thy
rename : src/HOL/Probability/Regularity.thy => src/HOL/Multivariate_Analysis/Regularity.thy
rename : src/HOL/Probability/Set_Integral.thy => src/HOL/Multivariate_Analysis/Set_Integral.thy
rename : src/HOL/Probability/Sigma_Algebra.thy => src/HOL/Multivariate_Analysis/Sigma_Algebra.thy
rename : src/HOL/Probability/measurable.ML => src/HOL/Multivariate_Analysis/measurable.ML
extra : rebase_source : 30ab39c42165c1c5622833cf256065cbfff030f9


# ee163328 29-Jul-2016 wenzelm <none@none>

more accurate cong del;
tuned proofs;


# a2bc0021 25-Apr-2016 wenzelm <none@none>

eliminated old 'def';
tuned comments;


# 79d3be54 14-Apr-2016 hoelzl <none@none>

Probability: move emeasure and nn_integral from ereal to ennreal

--HG--
extra : rebase_source : 5f2ac8a84abb43927a58086db8bbe10e190b2e77


# 35f7dccd 23-Feb-2016 nipkow <none@none>

more canonical names


# 8e83c9d2 07-Dec-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 3f106d8a 10-Nov-2015 paulson <lp15@cam.ac.uk>

Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.


# 5012105f 13-Sep-2015 wenzelm <none@none>

tuned proofs -- less legacy;


# 5b7d639c 25-Jun-2015 wenzelm <none@none>

tuned proofs;


# d6db773a 11-Apr-2015 paulson <lp15@cam.ac.uk>

Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.


# f8e9ab7b 02-Nov-2014 wenzelm <none@none>

modernized header;


# bf4e83d3 28-Jun-2014 haftmann <none@none>

fact consolidation


# 69ece7a6 13-Jun-2014 hoelzl <none@none>

properties of normal distributed random variables (by Sudeep Kanav)


# 33db321f 12-Jun-2014 hoelzl <none@none>

properties of Erlang and exponentially distributed random variables (by Sudeep Kanav)

--HG--
extra : rebase_source : b821e7a52658fa32f598433901729ddc5fc949dd


# a876535b 03-Jun-2014 hoelzl <none@none>

use 0 as integral-value for non-integrable functions, simplify a couple of rewrite rules

--HG--
extra : rebase_source : 768e923634e619b4e9e3d904c01eda79077c3963


# f281533d 19-May-2014 hoelzl <none@none>

renamed positive_integral to nn_integral

--HG--
extra : rebase_source : e7a432bee0942b6330cadfd1eb5da8e326238e06


# ab027a86 19-May-2014 hoelzl <none@none>

fixed document generation for HOL-Probability


# 1a8832ef 18-May-2014 hoelzl <none@none>

introduce Bochner integral: generalizes Lebesgue integral from real-valued function to functions on real-normed vector spaces

--HG--
rename : src/HOL/Probability/Lebesgue_Integration.thy => src/HOL/Probability/Nonnegative_Lebesgue_Integration.thy


# 66804330 14-Apr-2014 hoelzl <none@none>

added divide_nonneg_nonneg and co; made it a simp rule

--HG--
extra : rebase_source : 998eadb7cfbf8720cf961ac2e149ce4537557a47


# 5723122d 12-Apr-2014 nipkow <none@none>

made mult_pos_pos a simp rule


# 838cbeac 11-Apr-2014 nipkow <none@none>

made divide_pos_pos a simp rule


# a444e184 11-Apr-2014 nipkow <none@none>

made mult_nonneg_nonneg a simp rule

--HG--
extra : rebase_source : 3f70ac991fa0f02839309ce9b8f418ff53f87c36


# 77b90a1d 09-Apr-2014 hoelzl <none@none>

revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules


# 36a1e2cc 03-Apr-2014 paulson <lp15@cam.ac.uk>

removing simprule status for divide_minus_left and divide_minus_right


# 88cc155c 15-Mar-2014 haftmann <none@none>

more complete set of lemmas wrt. image and composition


# 7237bdd9 02-Sep-2013 wenzelm <none@none>

tuned proofs -- clarified flow of facts wrt. calculation;


# 06329277 13-Aug-2013 wenzelm <none@none>

standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;


# 1cbdc003 07-Dec-2012 hoelzl <none@none>

add exponential and uniform distributions


# ba5f9f86 27-Nov-2012 immler <none@none>

qualified interpretation of sigma_algebra, to avoid name clashes

--HG--
extra : rebase_source : aaeab4e40463c23ef5a5a07ee360db0335376105


# fde36cfd 02-Nov-2012 hoelzl <none@none>

use measurability prover


# e7b50b43 02-Nov-2012 hoelzl <none@none>

add measurability prover; add support for Borel sets


# 9a923f72 02-Nov-2012 hoelzl <none@none>

for the product measure it is enough if only one measure is sigma-finite


# 082e9e56 11-Oct-2012 hoelzl <none@none>

cleanup borel_measurable_positive_integral_(fst|snd)


# 3bd1870d 09-Oct-2012 hoelzl <none@none>

add finite entropy


# a8bf5036 09-Oct-2012 hoelzl <none@none>

continuous version of mutual_information_eq_entropy_conditional_entropy


# bf7737b4 09-Oct-2012 hoelzl <none@none>

remove unnecessary assumption from conditional_entropy_eq


# 4b56688a 09-Oct-2012 hoelzl <none@none>

alternative definition of conditional entropy


# 1c16ea97 09-Oct-2012 hoelzl <none@none>

remove unneeded assumption from conditional_entropy_generic_eq


# 2cfd7071 09-Oct-2012 hoelzl <none@none>

show and use distributed_swap and distributed_jointI


# 992a23c0 09-Oct-2012 hoelzl <none@none>

rule to show that conditional mutual information is non-negative in the continuous case


# 78bc643f 09-Oct-2012 hoelzl <none@none>

continuous version of entropy_le


# 20cd5b52 09-Oct-2012 hoelzl <none@none>

simplified entropy_uniform


# 73a18021 09-Oct-2012 hoelzl <none@none>

tuned product measurability


# 11c87ed0 22-Apr-2012 hoelzl <none@none>

reworked Probability theory

--HG--
extra : rebase_source : 04bef352ab6c7feafcf64ecca49fecffac43bb41


# 95291102 13-Mar-2012 wenzelm <none@none>

prefer abs_def over def_raw;


# 33cd0191 28-Feb-2012 wenzelm <none@none>

avoid undeclared variables in let bindings;
tuned proofs;


# f083f9a4 07-Dec-2011 hoelzl <none@none>

remove unnecessary sublocale instantiations in HOL-Probability (for clarity and speedup); remove Infinite_Product_Measure.product_prob_space which was a duplicate of Probability_Measure.product_prob_space


# d5c9d81f 01-Dec-2011 hoelzl <none@none>

moved theorems about distribution to the definition; removed oopsed-lemma


# ccb77667 01-Dec-2011 hoelzl <none@none>

remove duplicate theorem setsum_real_distribution


# ad9e459c 11-Sep-2011 nipkow <none@none>

new fastforce replacing fastsimp - less confusing name


# 7f546ab9 19-Jul-2011 hoelzl <none@none>

Rename extreal => ereal

--HG--
rename : src/HOL/Library/Extended_Reals.thy => src/HOL/Library/Extended_Real.thy


# 78fb9bbf 27-Jun-2011 hoelzl <none@none>

move conditional expectation to its own theory file


# 04d61436 09-Jun-2011 hoelzl <none@none>

lemma: independence is equal to mutual information = 0


# de7c70f0 29-Mar-2011 hoelzl <none@none>

rename Probability_Space to Probability_Measure

--HG--
rename : src/HOL/Probability/Probability_Space.thy => src/HOL/Probability/Probability_Measure.thy


# 78b9d3de 22-Mar-2011 hoelzl <none@none>

standardized headers


# 6c82f941 14-Mar-2011 hoelzl <none@none>

reworked Probability theory: measures are not type restricted to positive extended reals


# cc8cb183 23-Feb-2011 hoelzl <none@none>

add lemma KL_divergence_vimage, mutual_information_generic


# 93b9a16c 01-Feb-2011 hoelzl <none@none>

the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
changed syntax for simple_function, simple_integral, positive_integral, integral and RN_deriv.
introduced binder variants for simple_integral, positive_integral and integral.


# 244d6114 24-Jan-2011 hoelzl <none@none>

use pre-image measure, instead of image


# 3d40d3d4 29-Dec-2010 wenzelm <none@none>

explicit file specifications -- avoid secondary load path;


# cdf55c33 08-Dec-2010 hoelzl <none@none>

cleanup bijectivity btw. product spaces and pairs


# 8dce21d4 03-Dec-2010 hoelzl <none@none>

it is known as the extended reals, not the infinite reals

--HG--
rename : src/HOL/Probability/Positive_Infinite_Real.thy => src/HOL/Probability/Positive_Extended_Real.thy


# 481ae947 01-Dec-2010 hoelzl <none@none>

Support product spaces on sigma finite measures.
Introduce the almost everywhere quantifier.
Introduce 'morphism' theorems for most constants.
Prove uniqueness of measures on cut stable generators.
Prove uniqueness of the Radon-Nikodym derivative.
Removed misleading suffix from borel_space and lebesgue_space.
Use product spaces to introduce Fubini on the Lebesgue integral.
Combine Euclidean_Lebesgue and Lebesgue_Measure.
Generalize theorems about mutual information and entropy to arbitrary probability spaces.
Remove simproc mult_log as it does not work with interpretations.
Introduce completion of measure spaces.
Change type of sigma.
Introduce dynkin systems.

--HG--
rename : src/HOL/Probability/Borel.thy => src/HOL/Probability/Borel_Space.thy


# 5b59da77 13-Sep-2010 nipkow <none@none>

renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI


# bb8268b1 07-Sep-2010 nipkow <none@none>

expand_fun_eq -> ext_iff
expand_set_eq -> set_ext_iff
Naming in line now with multisets


# 2890c985 02-Sep-2010 hoelzl <none@none>

Moved lemmas to appropriate locations


# 9c9ff2a8 02-Sep-2010 hoelzl <none@none>

move lemmas to correct theory files


# 2eca6769 23-Aug-2010 hoelzl <none@none>

Rewrite the Probability theory.

Introduced pinfreal as real numbers with infinity.
Use pinfreal as value for measures.
Introduces Lebesgue Measure based on the integral in Multivariate Analysis.
Proved Radon Nikodym for arbitrary sigma finite measure spaces.

--HG--
rename : src/HOL/Probability/Lebesgue.thy => src/HOL/Probability/Lebesgue_Integration.thy


# 0dd4f9c2 04-May-2010 hoelzl <none@none>

Corrected imports; better approximation of dependencies.


# bb4b3c35 03-May-2010 hoelzl <none@none>

Cleanup information theory


# 2921aff7 03-May-2010 hoelzl <none@none>

Moved Convex theory to library.


# 9a8190f3 07-Apr-2010 hoelzl <none@none>

Added Information theory and Example: dining cryptographers