Skip to content

Commit

Permalink
feat(Data/Set/Pairwise/Basic): pairwise disjoint sets and subsingleto…
Browse files Browse the repository at this point in the history
…ns (#11629)

Add a lemma giving a characterization of pairwise disjoint sets in terms of each value lying in at most one set:

```lean
lemma subsingleton_setOf_mem_iff_pairwise_disjoint {f : ι → Set α} :
    (∀ a, {i | a ∈ f i}.Subsingleton) ↔ Pairwise (Disjoint on f) :=
```

From AperiodicMonotilesLean.
  • Loading branch information
jsm28 committed Apr 4, 2024
1 parent 2c870c1 commit 9740087
Showing 1 changed file with 5 additions and 0 deletions.
5 changes: 5 additions & 0 deletions Mathlib/Data/Set/Pairwise/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -458,3 +458,8 @@ lemma exists_lt_mem_inter_of_not_pairwise_disjoint [LinearOrder ι]
theorem pairwise_disjoint_fiber (f : ι → α) : Pairwise (Disjoint on fun a : α => f ⁻¹' {a}) :=
pairwise_univ.1 <| Set.pairwiseDisjoint_fiber f univ
#align pairwise_disjoint_fiber pairwise_disjoint_fiber

lemma subsingleton_setOf_mem_iff_pairwise_disjoint {f : ι → Set α} :
(∀ a, {i | a ∈ f i}.Subsingleton) ↔ Pairwise (Disjoint on f) :=
fun h _ _ hij ↦ disjoint_left.2 fun a hi hj ↦ hij (h a hi hj),
fun h _ _ hx _ hy ↦ by_contra fun hne ↦ disjoint_left.1 (h hne) hx hy⟩

0 comments on commit 9740087

Please sign in to comment.