src/HOL/Probability/Probability.thy
author haftmann
Thu, 19 Jul 2012 19:38:39 +0200
changeset 48357 828ace4f75ab
parent 47694 05663f75964c
child 50087 635d73673b5e
permissions -rw-r--r--
removed ML module DSeq which was a part of the ancient code generator (cf. 58e33a125f32)

theory Probability
imports
  Complete_Measure
  Probability_Measure
  Infinite_Product_Measure
  Independent_Family
  Information
begin

end