Skip to content

Commit 00056bc

Browse files
committed
chore: bump std to leanprover/lean4#429 (#8990)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent 8ec98e4 commit 00056bc

File tree

3 files changed

+3
-8
lines changed

3 files changed

+3
-8
lines changed

Mathlib/Data/List/Perm.lean

Lines changed: 1 addition & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -229,14 +229,9 @@ lemma subperm_iff : l₁ <+~ l₂ ↔ ∃ l, l ~ l₂ ∧ l₁ <+ l := by
229229
obtain ⟨l', h₂⟩ := h₂.exists_perm_append
230230
exact ⟨l₁ ++ l', (h₂.trans (h₁.append_right _)).symm, (prefix_append _ _).sublist⟩
231231

232-
-- This is now in `Std`, but apparently misnamed as `List.subperm_singleton_iff`.
233-
lemma singleton_subperm_iff : [a] <+~ l ↔ a ∈ l :=
234-
fun ⟨s, hla, h⟩ ↦ by rwa [perm_singleton.1 hla, singleton_sublist] at h,
235-
fun h ↦ ⟨[a], perm_rfl, singleton_sublist.2 h⟩⟩
236232
#align list.subperm_singleton_iff List.singleton_subperm_iff
237233

238-
-- The prime could be removed if `List.subperm_singleton_iff` is renamed in Std.
239-
@[simp] lemma subperm_singleton_iff' : l <+~ [a] ↔ l = [] ∨ l = [a] := by
234+
@[simp] lemma subperm_singleton_iff : l <+~ [a] ↔ l = [] ∨ l = [a] := by
240235
constructor
241236
· rw [subperm_iff]
242237
rintro ⟨s, hla, h⟩

Mathlib/Data/Multiset/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -621,7 +621,7 @@ theorem singleton_le {a : α} {s : Multiset α} : {a} ≤ s ↔ a ∈ s :=
621621

622622
@[simp] lemma le_singleton : s ≤ {a} ↔ s = 0 ∨ s = {a} :=
623623
Quot.induction_on s fun l ↦ by simp only [cons_zero, ← coe_singleton, quot_mk_to_coe'', coe_le,
624-
coe_eq_zero, coe_eq_coe, perm_singleton, subperm_singleton_iff']
624+
coe_eq_zero, coe_eq_coe, perm_singleton, subperm_singleton_iff]
625625

626626
@[simp] lemma lt_singleton : s < {a} ↔ s = 0 := by
627627
simp only [lt_iff_le_and_ne, le_singleton, or_and_right, Ne.def, and_not_self, or_false,

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": "604b4078d46104d4144a87ebf4c2dae581cb704a",
7+
"rev": "483fd2846f9fe5107011ece0cc3d8d88af1a8603",
88
"name": "std",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",

0 commit comments

Comments
 (0)