src/HOL/Probability/ex/Koepf_Duermuth_Countermeasure.thy
changeset 41413 64cd30d6b0b8
parent 41023 9118eb4eb8dc
child 41689 3e39b0e730d6
equal deleted inserted replaced
41412:35f30e07fe0d 41413:64cd30d6b0b8
     1 (* Author: Johannes Hoelzl, TU Muenchen *)
     1 (* Author: Johannes Hoelzl, TU Muenchen *)
     2 
     2 
     3 header {* Formalization of a Countermeasure by Koepf & Duermuth 2009 *}
     3 header {* Formalization of a Countermeasure by Koepf & Duermuth 2009 *}
     4 
     4 
     5 theory Koepf_Duermuth_Countermeasure
     5 theory Koepf_Duermuth_Countermeasure
     6   imports Information Permutation
     6   imports Information "~~/src/HOL/Library/Permutation"
     7 begin
     7 begin
     8 
     8 
     9 lemma
     9 lemma
    10   fixes p u :: "'a \<Rightarrow> real"
    10   fixes p u :: "'a \<Rightarrow> real"
    11   assumes "1 < b"
    11   assumes "1 < b"