Skip to content

Commit

Permalink
chore(data/finset/basic): erase_inj_on (#6769)
Browse files Browse the repository at this point in the history
Quick follow-up to #6737
  • Loading branch information
pechersky committed Mar 19, 2021
1 parent 2d2929f commit c65146d
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/data/finset/basic.lean
Expand Up @@ -906,6 +906,9 @@ begin
simp,
end

lemma erase_inj_on (s : finset α) : set.inj_on s.erase s :=
λ _ _ _ _, (erase_inj s ‹_›).mp

/-! ### sdiff -/

/-- `s \ t` is the set consisting of the elements of `s` that are not in `t`. -/
Expand Down

0 comments on commit c65146d

Please sign in to comment.