src/HOL/Probability/Probability.thy
author wenzelm
Mon, 23 Nov 2015 16:57:01 +0100
changeset 61737 b91b1ebfc8a0
parent 61359 e985b52c3eb3
child 62083 7582b39f51ed
permissions -rw-r--r--
bundle main sources read-only, to avoid accidental editing of imported theories etc.;

(*  Title:      HOL/Probability/Probability.thy
    Author:     Johannes Hölzl, TU München
*)

theory Probability
imports
  Discrete_Topology
  Complete_Measure
  Projective_Limit
  Independent_Family
  Distributions
  Probability_Mass_Function
  Stream_Space
  Embed_Measure
begin

end