Skip to content

Commit

Permalink
Update finset.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 committed Apr 26, 2018
1 parent c995f62 commit 009ff9b
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions data/finset.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1014,10 +1014,10 @@ theorem disjoint_of_subset_left {s t u : finset α} (h : s ⊆ u) (d : disjoint
theorem disjoint_of_subset_right {s t u : finset α} (h : t ⊆ u) (d : disjoint s u) : disjoint s t
| x m m₁ := d m (h m₁)

@[simp] theorem empty_disjoint (s : finset α) : disjoint ∅ s
@[simp] theorem disjoint_empty_left (s : finset α) : disjoint ∅ s
| a := (not_mem_empty a).elim

@[simp] theorem disjoint_empty (s : finset α) : disjoint s ∅ :=
@[simp] theorem disjoint_empty_right (s : finset α) : disjoint s ∅ :=
disjoint_comm.1 (empty_disjoint _)

@[simp] theorem singleton_disjoint {s : finset α} {a : α} : disjoint (singleton a) s ↔ a ∉ s :=
Expand Down

0 comments on commit 009ff9b

Please sign in to comment.