src/HOL/Analysis/Measure_Space.thy
changeset 70614 6a2c982363e9
parent 70532 fcf3b891ccb1
child 70722 ae2528273eeb
--- a/src/HOL/Analysis/Measure_Space.thy	Sun Aug 25 22:17:24 2019 +0200
+++ b/src/HOL/Analysis/Measure_Space.thy	Tue Aug 27 17:08:51 2019 +0200
@@ -1184,9 +1184,6 @@
   "(\<And>N. N \<in> I \<Longrightarrow> AE x in M. P N x) \<Longrightarrow> countable I \<Longrightarrow> AE x in M. \<forall>N \<in> I. P N x"
   unfolding AE_ball_countable by simp
 
-lemma pairwise_alt: "pairwise R S \<longleftrightarrow> (\<forall>x\<in>S. \<forall>y\<in>S-{x}. R x y)"
-  by (auto simp add: pairwise_def)
-
 lemma AE_pairwise: "countable F \<Longrightarrow> pairwise (\<lambda>A B. AE x in M. R x A B) F \<longleftrightarrow> (AE x in M. pairwise (R x) F)"
   unfolding pairwise_alt by (simp add: AE_ball_countable)