src/HOL/Probability/Probability.thy
author blanchet
Wed, 01 Jun 2011 10:29:43 +0200
changeset 43133 eb8ec21c9a48
parent 42902 e8dbf90a2f3b
child 43556 0d78c8d31d0d
permissions -rw-r--r--
fixed Isabelle version of lightweight tag theorem, using "Thm.trivial" not "Thm.assume"

theory Probability
imports
  Complete_Measure
  Probability_Measure
  Infinite_Product_Measure
  Independent_Family
  Information
  "ex/Dining_Cryptographers"
  "ex/Koepf_Duermuth_Countermeasure"
begin
end