src/HOL/Probability/Probability.thy
author blanchet
Thu, 12 May 2011 15:29:19 +0200
changeset 42744 59753d5448e0
parent 42148 d596e7bb251f
child 42861 16375b493b64
permissions -rw-r--r--
added "SMT." qualifier for constant to make it possible to reload "smt_monomorph.ML" from outside the "SMT" theory (for experiments) -- this is also consistent with the other SMT constants mentioned in this source file

theory Probability
imports
  Complete_Measure
  Lebesgue_Measure
  Probability_Measure
  Infinite_Product_Measure
  Information
  "ex/Dining_Cryptographers"
  "ex/Koepf_Duermuth_Countermeasure"
begin
end