Commit
This commit does not belong to any branch on this repository, and may belong to a fork outside of the repository.
feat(Data/Nat/Nth):
nth_mem_anti
(#19169)
Add another lemma for working with `Nat.nth`: ```lean lemma nth_mem_anti {a b : ℕ} (hab : a ≤ b) (h : p (nth p b)) : p (nth p a) := by ``` Feel free to golf if you see a simpler way of proving this.
- Loading branch information