src/HOL/Probability/Probability.thy
author haftmann
Tue, 11 May 2010 08:36:02 +0200
changeset 36811 4ab4aa5bee1c
parent 36080 0d9affa4e73c
child 40859 de0b30e6c2d2
permissions -rw-r--r--
renamed former Int.int_induct to Int.int_of_nat_induct, former Presburger.int_induct to Int.int_induct: is more conservative and more natural than the intermediate solution

theory Probability
imports
  Information
  "ex/Dining_Cryptographers"
begin

end