src/HOL/Probability/ex/Koepf_Duermuth_Countermeasure.thy
changeset 67399 eab6ce8368fa
parent 66804 3f9bb52082c4
child 70347 e5cd5471c18a
--- a/src/HOL/Probability/ex/Koepf_Duermuth_Countermeasure.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Probability/ex/Koepf_Duermuth_Countermeasure.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -194,7 +194,7 @@
 definition t :: "'observation list \<Rightarrow> 'observation \<Rightarrow> nat" where
   t_def2: "t seq obs = card { i. i < length seq \<and> seq ! i = obs}"
 
-lemma t_def: "t seq obs = length (filter (op = obs) seq)"
+lemma t_def: "t seq obs = length (filter ((=) obs) seq)"
   unfolding t_def2 length_filter_conv_card by (subst eq_commute) simp
 
 lemma card_T_bound: "card ((t\<circ>OB)`msgs) \<le> (n+1)^card observations"