src/HOL/Probability/Probability.thy
author wenzelm
Sun, 02 Sep 2012 14:02:05 +0200
changeset 49064 bd6cc0b911a1
parent 47694 05663f75964c
child 50087 635d73673b5e
permissions -rw-r--r--
maintain stable state of node entries from last round -- bypass slightly different Thm.join_theory_proofs;

theory Probability
imports
  Complete_Measure
  Probability_Measure
  Infinite_Product_Measure
  Independent_Family
  Information
begin

end