Skip to content

Commit

Permalink
fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Mar 4, 2024
1 parent 5a86dde commit bd7633c
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Data/Fin/Tuple/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -782,7 +782,7 @@ theorem insertNth_apply_succAbove (i : Fin (n + 1)) (x : α i) (p : ∀ j, α (i
rw [castPred_succAbove _ _ hlt] at hk; cases hk
intro; rfl
· generalize_proofs H₁ H₂; revert H₂
generalize hk : pred ((succAboveEmb i).toEmbedding j) H₁ = k
generalize hk : pred (succAbove i j) H₁ = k
erw [pred_succAbove _ _ (le_of_not_lt hlt)] at hk; cases hk
intro; rfl
#align fin.insert_nth_apply_succ_above Fin.insertNth_apply_succAbove
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/List/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1430,7 +1430,7 @@ theorem modifyNth_eq_set (f : α → α) :
| 0, l => by cases l <;> rfl
| n + 1, [] => rfl
| n + 1, b :: l =>
(congr_arg (cons b) (modifyNth_eq_set f n l)).trans <| by cases get? l n <;> rfl
(congr_arg (cons b) (modifyNth_eq_set f n l)).trans <| by cases h : get? l n <;> simp [h]
#align list.modify_nth_eq_update_nth List.modifyNth_eq_set

#align list.nth_modify_nth List.get?_modifyNth
Expand Down

0 comments on commit bd7633c

Please sign in to comment.