src/HOL/Probability/Probability.thy
author hoelzl
Wed, 01 Dec 2010 19:20:30 +0100
changeset 40859 de0b30e6c2d2
parent 36080 0d9affa4e73c
child 41689 3e39b0e730d6
permissions -rw-r--r--
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.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
33536
fd28b7399f2b eliminated hard tabulators;
wenzelm
parents: 33271
diff changeset
     1
theory Probability
36080
0d9affa4e73c Added Information theory and Example: dining cryptographers
hoelzl
parents: 35833
diff changeset
     2
imports
0d9affa4e73c Added Information theory and Example: dining cryptographers
hoelzl
parents: 35833
diff changeset
     3
  Information
0d9affa4e73c Added Information theory and Example: dining cryptographers
hoelzl
parents: 35833
diff changeset
     4
  "ex/Dining_Cryptographers"
33271
7be66dee1a5a New theory Probability, which contains a development of measure theory
paulson
parents:
diff changeset
     5
begin
7be66dee1a5a New theory Probability, which contains a development of measure theory
paulson
parents:
diff changeset
     6
end