Skip to content

Commit

Permalink
deprecation
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 20, 2024
1 parent dadfebc commit 33e7503
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Testing/Plausible/Functions.lean
Original file line number Diff line number Diff line change
Expand Up @@ -202,7 +202,7 @@ theorem List.applyId_zip_eq [DecidableEq α] {xs ys : List α} (h₀ : List.Nodu
simp only [getElem?_cons_succ, zip_cons_cons, applyId_cons] at h₂ ⊢
rw [if_neg]
· apply xs_ih <;> solve_by_elim [Nat.succ.inj]
· apply h₀; apply List.getElem?_mem h₂
· apply h₀; apply List.mem_of_getElem? h₂

theorem applyId_mem_iff [DecidableEq α] {xs ys : List α} (h₀ : List.Nodup xs) (h₁ : xs ~ ys)
(x : α) : List.applyId.{u} (xs.zip ys) x ∈ ys ↔ x ∈ xs := by
Expand Down

0 comments on commit 33e7503

Please sign in to comment.