src/HOL/Probability/Probability.thy
author haftmann
Thu, 01 Jul 2010 16:54:44 +0200
changeset 37678 0040bafffdef
parent 36080 0d9affa4e73c
child 40859 de0b30e6c2d2
permissions -rw-r--r--
"prod" and "sum" replace "*" and "+" respectively

theory Probability
imports
  Information
  "ex/Dining_Cryptographers"
begin

end