Skip to content

Commit d4e8dd2

Browse files
kim-emnomeatadigama0
committed
chore: update dependencies (#12792)
Co-authored-by: Joachim Breitner <mail@joachim-breitner.de> Co-authored-by: Mario Carneiro <di.gama@gmail.com>
1 parent daade17 commit d4e8dd2

File tree

3 files changed

+18
-13
lines changed

3 files changed

+18
-13
lines changed

Mathlib/Data/List/OfFn.lean

Lines changed: 13 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -36,23 +36,28 @@ namespace List
3636

3737
#noalign list.length_of_fn_aux
3838

39+
@[simp]
40+
theorem length_ofFn_go {n} (f : Fin n → α) (i j h) : length (ofFn.go f i j h) = i := by
41+
induction i generalizing j <;> simp_all [ofFn.go]
42+
3943
/-- The length of a list converted from a function is the size of the domain. -/
4044
@[simp]
4145
theorem length_ofFn {n} (f : Fin n → α) : length (ofFn f) = n := by
42-
simp [ofFn]
46+
simp [ofFn, length_ofFn_go]
4347
#align list.length_of_fn List.length_ofFn
4448

4549
#noalign list.nth_of_fn_aux
4650

51+
theorem get_ofFn_go {n} (f : Fin n → α) (i j h) (k) (hk) :
52+
get (ofFn.go f i j h) ⟨k, hk⟩ = f ⟨j + k, by simp at hk; omega⟩ := by
53+
let i+1 := i
54+
cases k <;> simp [ofFn.go, get_ofFn_go (i := i)]
55+
congr 2; omega
56+
4757
-- Porting note (#10756): new theorem
4858
@[simp]
4959
theorem get_ofFn {n} (f : Fin n → α) (i) : get (ofFn f) i = f (Fin.cast (by simp) i) := by
50-
have := Array.getElem_ofFn f i (by simpa using i.2)
51-
cases' i with i hi
52-
simp only [getElem, Array.get] at this
53-
simp only [Fin.cast_mk]
54-
rw [← this]
55-
congr
60+
cases i; simp [ofFn, get_ofFn_go]
5661

5762
/-- The `n`th element of a list -/
5863
@[simp]
@@ -114,7 +119,7 @@ theorem ofFn_zero (f : Fin 0 → α) : ofFn f = [] :=
114119
theorem ofFn_succ {n} (f : Fin (succ n) → α) : ofFn f = f 0 :: ofFn fun i => f i.succ :=
115120
ext_get (by simp) (fun i hi₁ hi₂ => by
116121
cases i
117-
· simp
122+
· simp; rfl
118123
· simp)
119124
#align list.of_fn_succ List.ofFn_succ
120125

Mathlib/LinearAlgebra/ExteriorAlgebra/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -334,8 +334,8 @@ theorem ιMulti_zero_apply (v : Fin 0 → M) : ιMulti R 0 v = 1 :=
334334

335335
@[simp]
336336
theorem ιMulti_succ_apply {n : ℕ} (v : Fin n.succ → M) :
337-
ιMulti R _ v = ι R (v 0) * ιMulti R _ (Matrix.vecTail v) :=
338-
(congr_arg List.prod (List.ofFn_succ _)).trans List.prod_cons
337+
ιMulti R _ v = ι R (v 0) * ιMulti R _ (Matrix.vecTail v) := by
338+
simp [ιMulti, Matrix.vecTail]
339339
#align exterior_algebra.ι_multi_succ_apply ExteriorAlgebra.ιMulti_succ_apply
340340

341341
theorem ιMulti_succ_curryLeft {n : ℕ} (m : M) :

lake-manifest.json

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@
44
[{"url": "https://github.com/leanprover-community/batteries",
55
"type": "git",
66
"subDir": null,
7-
"rev": "56d2e4ee226603eb6b90b05f6b944bde42672cd5",
7+
"rev": "cac5bff36ff3c339d8fdb0d1506ec789ce57a6fd",
88
"name": "batteries",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",
@@ -22,7 +22,7 @@
2222
{"url": "https://github.com/leanprover-community/aesop",
2323
"type": "git",
2424
"subDir": null,
25-
"rev": "2225b0e4a3528da20499e2304b521e0c4c2a4563",
25+
"rev": "093226b2a8c0cdeac12f1b4786827c67c673b4fb",
2626
"name": "aesop",
2727
"manifestFile": "lake-manifest.json",
2828
"inputRev": "master",
@@ -49,7 +49,7 @@
4949
{"url": "https://github.com/leanprover-community/import-graph.git",
5050
"type": "git",
5151
"subDir": null,
52-
"rev": "c46d22bbe4f8363c0829ce0eb48a95012cdc0d79",
52+
"rev": "e9fb4ecc5d718eb36faae5308880cd3f243788df",
5353
"name": "importGraph",
5454
"manifestFile": "lake-manifest.json",
5555
"inputRev": "main",

0 commit comments

Comments
 (0)