src/HOL/Probability/Probability.thy
author wenzelm
Fri, 20 Aug 2010 11:47:33 +0200
changeset 38566 8176107637ce
parent 36080 0d9affa4e73c
child 40859 de0b30e6c2d2
permissions -rw-r--r--
Branches.overlapping: proper treatment of stop_range that overlaps with end; Markup_Tree.select: allow singularity in parent range specification;
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
7be66dee1a5a New theory Probability, which contains a development of measure theory
paulson
parents:
diff changeset
     7
end