Skip to content

Commit

Permalink
chore: fix name of Multiset.Nodup.filterMap (#1736)
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Jan 21, 2023
1 parent 8e030b6 commit d96e4c3
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions Mathlib/Data/Multiset/Nodup.lean
Expand Up @@ -197,10 +197,10 @@ protected theorem Nodup.sigma {σ : α → Type _} {t : ∀ a, Multiset (σ a)}
simpa [←funext hf] using List.Nodup.sigma
#align multiset.nodup.sigma Multiset.Nodup.sigma

protected theorem Nodup.filter_map (f : α → Option β) (H : ∀ a a' b, b ∈ f a → b ∈ f a' → a = a') :
protected theorem Nodup.filterMap (f : α → Option β) (H : ∀ a a' b, b ∈ f a → b ∈ f a' → a = a') :
Nodup s → Nodup (filterMap f s) :=
Quot.induction_on s fun _ => Nodup.filterMap H
#align multiset.nodup.filter_map Multiset.Nodup.filter_map
Quot.induction_on s fun _ => List.Nodup.filterMap H
#align multiset.nodup.filter_map Multiset.Nodup.filterMap

theorem nodup_range (n : ℕ) : Nodup (range n) :=
List.nodup_range _
Expand Down

0 comments on commit d96e4c3

Please sign in to comment.