Skip to content

Commit a6e8dce

Browse files
committed
chore(Data/Finset): remove deprecated lemma Finset.filter_mem_image_eq_image (#23054)
This has been deprecated for over 6 months and was blocking a (minor) import reduction.
1 parent b524d8d commit a6e8dce

File tree

4 files changed

+8
-6
lines changed

4 files changed

+8
-6
lines changed

Mathlib/Data/Finset/BooleanAlgebra.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ Copyright (c) 2017 Mario Carneiro. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Mario Carneiro
55
-/
6+
import Mathlib.Data.Finset.Basic
67
import Mathlib.Data.Finset.Image
78
import Mathlib.Data.Fintype.Defs
89

Mathlib/Data/Finset/Card.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ Copyright (c) 2015 Microsoft Corporation. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Leonardo de Moura, Jeremy Avigad
55
-/
6+
import Mathlib.Data.Finset.Basic
67
import Mathlib.Data.Finset.Image
78

89
/-!

Mathlib/Data/Finset/Fold.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ Copyright (c) 2017 Mario Carneiro. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Mario Carneiro
55
-/
6+
import Mathlib.Data.Finset.Basic
67
import Mathlib.Data.Finset.Image
78
import Mathlib.Data.Multiset.Fold
89

Mathlib/Data/Finset/Image.lean

Lines changed: 5 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,11 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Leonardo de Moura, Jeremy Avigad, Minchao Wu, Mario Carneiro
55
-/
66
import Mathlib.Data.Fin.Basic
7-
import Mathlib.Data.Finset.Basic
7+
import Mathlib.Data.Finset.Attach
8+
import Mathlib.Data.Finset.Disjoint
9+
import Mathlib.Data.Finset.Erase
10+
import Mathlib.Data.Finset.Filter
11+
import Mathlib.Data.Finset.Range
812
import Mathlib.Data.Finset.SymmDiff
913

1014
/-! # Image and map operations on finite sets
@@ -398,11 +402,6 @@ theorem filter_image {p : β → Prop} [DecidablePred p] :
398402
by rintro ⟨⟨x, h1, rfl⟩, h2⟩; exact ⟨x, ⟨h1, h2⟩, rfl⟩,
399403
by rintro ⟨x, ⟨h1, h2⟩, rfl⟩; exact ⟨⟨x, h1, rfl⟩, h2⟩⟩
400404

401-
@[deprecated filter_mem_eq_inter (since := "2024-09-15")]
402-
theorem filter_mem_image_eq_image (f : α → β) (s : Finset α) (t : Finset β) (h : ∀ x ∈ s, f x ∈ t) :
403-
(t.filter fun y => y ∈ s.image f) = s.image f := by
404-
rwa [filter_mem_eq_inter, inter_eq_right, image_subset_iff]
405-
406405
theorem fiber_nonempty_iff_mem_image {y : β} : (s.filter (f · = y)).Nonempty ↔ y ∈ s.image f := by
407406
simp [Finset.Nonempty]
408407

0 commit comments

Comments
 (0)