src/HOL/Probability/Probability.thy
author wenzelm
Mon, 11 Feb 2013 14:39:04 +0100
changeset 51085 d90218288d51
parent 50419 3177d0374701
child 57252 19b7ace1c5da
permissions -rw-r--r--
make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;

theory Probability
imports
  Discrete_Topology
  Complete_Measure
  Probability_Measure
  Infinite_Product_Measure
  Projective_Limit
  Independent_Family
  Information
  Distributions
begin

end