src/HOL/Probability/ex/Dining_Cryptographers.thy
changeset 56994 8d5e5ec1cac3
parent 53374 a14d2a854c02
child 57492 74bf65a1910a
equal deleted inserted replaced
56993:e5366291d6aa 56994:8d5e5ec1cac3
     6   by (unfold inj_on_def) blast
     6   by (unfold inj_on_def) blast
     7 
     7 
     8 lemma Ex1_eq: "\<exists>!x. P x \<Longrightarrow> P x \<Longrightarrow> P y \<Longrightarrow> x = y"
     8 lemma Ex1_eq: "\<exists>!x. P x \<Longrightarrow> P x \<Longrightarrow> P y \<Longrightarrow> x = y"
     9   by auto
     9   by auto
    10 
    10 
    11 section "Define the state space"
    11 subsection {* Define the state space *}
    12 
    12 
    13 text {*
    13 text {*
    14 
    14 
    15 We introduce the state space on which the algorithm operates.
    15 We introduce the state space on which the algorithm operates.
    16 
    16