Skip to content

Commit 11f79c5

Browse files
committed
chore: bump Std (#12256)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent 1d4a722 commit 11f79c5

File tree

2 files changed

+1
-7
lines changed

2 files changed

+1
-7
lines changed

Mathlib/Data/String/Lemmas.lean

Lines changed: 0 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -12,12 +12,6 @@ namespace String
1212
lemma congr_append : ∀ (a b : String), a ++ b = String.mk (a.data ++ b.data)
1313
| ⟨_⟩, ⟨_⟩ => rfl
1414

15-
@[simp] lemma length_append : ∀ (as bs : String), (as ++ bs).length = as.length + bs.length
16-
| ⟨as⟩, ⟨bs⟩ => by
17-
rw [congr_append]
18-
simp only [String.length]
19-
exact List.length_append as bs
20-
2115
@[simp] lemma length_replicate (n : ℕ) (c : Char) : (replicate n c).length = n := by
2216
simp only [String.length, String.replicate, List.length_replicate]
2317

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@
44
[{"url": "https://github.com/leanprover/std4",
55
"type": "git",
66
"subDir": null,
7-
"rev": "cb172855f1712a9e906e91f3e14541960562fb78",
7+
"rev": "e840c18f7334c751efbd4cfe531476e10c943cdb",
88
"name": "std",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",

0 commit comments

Comments
 (0)