src/HOL/Probability/Probability.thy
author hoelzl
Wed, 10 Oct 2012 12:12:33 +0200
changeset 49798 8d5668f73c42
parent 47694 05663f75964c
child 50087 635d73673b5e
permissions -rw-r--r--
induction prove for positive_integral_density

theory Probability
imports
  Complete_Measure
  Probability_Measure
  Infinite_Product_Measure
  Independent_Family
  Information
begin

end