Skip to content

Commit

Permalink
chore: drop unused changes
Browse files Browse the repository at this point in the history
  • Loading branch information
LeoDog896 committed Jan 6, 2025
1 parent 161e0a0 commit 2c1b10e
Showing 1 changed file with 0 additions and 2 deletions.
2 changes: 0 additions & 2 deletions Mathlib/Data/List/Nodup.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Kenny Lau
-/
import Mathlib.Data.List.Forall2
import Mathlib.Data.List.Lemmas
import Mathlib.Data.Set.Pairwise.Basic

/-!
Expand Down Expand Up @@ -389,7 +388,6 @@ theorem Nodup.take_eq_filter_mem [DecidableEq α] :
intro x hx
have : x ≠ b := fun h => (nodup_cons.1 hl).1 (h ▸ hx)
simp (config := {contextual := true}) [List.mem_filter, this, hx]

end List

theorem Option.toList_nodup : ∀ o : Option α, o.toList.Nodup
Expand Down

0 comments on commit 2c1b10e

Please sign in to comment.