src/HOL/Probability/Probability.thy
author blanchet
Mon, 21 May 2012 10:39:31 +0200
changeset 47944 e6b51fab96f7
parent 47694 05663f75964c
child 50087 635d73673b5e
permissions -rw-r--r--
added helper -- cf. SET616^5

theory Probability
imports
  Complete_Measure
  Probability_Measure
  Infinite_Product_Measure
  Independent_Family
  Information
begin

end