Skip to content

Commit

Permalink
chore: fix signature of perm_insertIdx (#6532)
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em authored Jan 4, 2025
1 parent d22233f commit 9dcbc33
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Init/Data/List/Perm.lean
Original file line number Diff line number Diff line change
Expand Up @@ -510,7 +510,7 @@ theorem Perm.eraseP (f : α → Bool) {l₁ l₂ : List α}
refine (IH₁ H).trans (IH₂ ((p₁.pairwise_iff ?_).1 H))
exact fun h h₁ h₂ => h h₂ h₁

theorem perm_insertIdx [DecidableEq α] {α} (x : α) (l : List α) {n} (h : n ≤ l.length) :
theorem perm_insertIdx {α} (x : α) (l : List α) {n} (h : n ≤ l.length) :
insertIdx n x l ~ x :: l := by
induction l generalizing n with
| nil =>
Expand Down

0 comments on commit 9dcbc33

Please sign in to comment.