src/HOL/Probability/Probability.thy
author nipkow
Mon, 01 Aug 2011 12:08:53 +0200
changeset 44045 2814ff2a6e3e
parent 43556 0d78c8d31d0d
child 45713 badee348c5fb
permissions -rw-r--r--
infrastructure for attaching names to hypothesis in cases; realised via the same tag mechanism as case names
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
41689
3e39b0e730d6 the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents: 40859
diff changeset
     3
  Complete_Measure
42148
d596e7bb251f rename Probability_Space to Probability_Measure
hoelzl
parents: 42147
diff changeset
     4
  Probability_Measure
42147
61d5d50ca74c add infinite product measure
hoelzl
parents: 41981
diff changeset
     5
  Infinite_Product_Measure
42861
16375b493b64 Add formalization of probabilistic independence for families of sets
hoelzl
parents: 42148
diff changeset
     6
  Independent_Family
43556
0d78c8d31d0d move conditional expectation to its own theory file
hoelzl
parents: 42902
diff changeset
     7
  Conditional_Probability
36080
0d9affa4e73c Added Information theory and Example: dining cryptographers
hoelzl
parents: 35833
diff changeset
     8
  Information
0d9affa4e73c Added Information theory and Example: dining cryptographers
hoelzl
parents: 35833
diff changeset
     9
  "ex/Dining_Cryptographers"
41689
3e39b0e730d6 the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents: 40859
diff changeset
    10
  "ex/Koepf_Duermuth_Countermeasure"
33271
7be66dee1a5a New theory Probability, which contains a development of measure theory
paulson
parents:
diff changeset
    11
begin
7be66dee1a5a New theory Probability, which contains a development of measure theory
paulson
parents:
diff changeset
    12
end