src/HOL/Probability/Probability.thy
author blanchet
Wed, 17 Mar 2010 12:01:01 +0100
changeset 35808 df56c1b1680f
parent 35582 b16d99a72dc9
child 35833 7b7ae5aa396d
permissions -rw-r--r--
fix typo in "nitpick_choice_spec" attribute name (singular, not plural)
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
33536
fd28b7399f2b eliminated hard tabulators;
wenzelm
parents: 33271
diff changeset
     1
theory Probability
35582
b16d99a72dc9 Add Lebesgue integral and probability space.
hoelzl
parents: 33544
diff changeset
     2
imports Probability_Space
33271
7be66dee1a5a New theory Probability, which contains a development of measure theory
paulson
parents:
diff changeset
     3
begin
7be66dee1a5a New theory Probability, which contains a development of measure theory
paulson
parents:
diff changeset
     4
7be66dee1a5a New theory Probability, which contains a development of measure theory
paulson
parents:
diff changeset
     5
end