src/HOL/Probability/Probability.thy
author hoelzl
Mon, 14 Mar 2011 14:37:49 +0100
changeset 41981 cdf7693bbe08
parent 41689 3e39b0e730d6
child 42147 61d5d50ca74c
permissions -rw-r--r--
reworked Probability theory: measures are not type restricted to positive extended reals

theory Probability
imports
  Complete_Measure
  Lebesgue_Measure
  Information
  "ex/Dining_Cryptographers"
  "ex/Koepf_Duermuth_Countermeasure"
begin
end