Skip to content

Commit fdf57b0

Browse files
kim-emdigama0
andcommitted
chore: bump Std to match leanprover-community/batteries#448 (#9044)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com> Co-authored-by: Mario Carneiro <di.gama@gmail.com>
1 parent a5732e8 commit fdf57b0

File tree

4 files changed

+8
-8
lines changed

4 files changed

+8
-8
lines changed

Mathlib/Data/List/Basic.lean

Lines changed: 4 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -247,12 +247,13 @@ theorem singleton_eq (x : α) : ({x} : List α) = [x] :=
247247
rfl
248248
#align list.singleton_eq List.singleton_eq
249249

250-
theorem insert_neg [DecidableEq α] {x : α} {l : List α} (h : x ∉ l) : Insert.insert x l = x :: l :=
251-
if_neg h
250+
theorem insert_neg [DecidableEq α] {x : α} {l : List α} (h : x ∉ l) :
251+
Insert.insert x l = x :: l :=
252+
insert_of_not_mem h
252253
#align list.insert_neg List.insert_neg
253254

254255
theorem insert_pos [DecidableEq α] {x : α} {l : List α} (h : x ∈ l) : Insert.insert x l = l :=
255-
if_pos h
256+
insert_of_mem h
256257
#align list.insert_pos List.insert_pos
257258

258259
theorem doubleton_eq [DecidableEq α] {x y : α} (h : x ≠ y) : ({x, y} : List α) = [x, y] := by

Mathlib/Data/List/Infix.lean

Lines changed: 3 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -469,9 +469,10 @@ theorem insert_nil (a : α) : insert a nil = [a] :=
469469
rfl
470470
#align list.insert_nil List.insert_nil
471471

472-
theorem insert.def (a : α) (l : List α) : insert a l = if a ∈ l then l else a :: l :=
472+
theorem insert_eq_ite (a : α) (l : List α) : insert a l = if a ∈ l then l else a :: l := by
473+
simp only [← elem_iff]
473474
rfl
474-
#align list.insert.def List.insert.def
475+
#align list.insert.def List.insert_eq_ite
475476

476477
#align list.insert_of_mem List.insert_of_mem
477478
#align list.insert_of_not_mem List.insert_of_not_mem

Mathlib/Logic/Basic.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1217,8 +1217,6 @@ protected theorem Ne.ite_ne_right_iff (h : a ≠ b) : ite P a b ≠ b ↔ P :=
12171217

12181218
variable (P Q a b)
12191219

1220-
/-- A `dite` whose results do not actually depend on the condition may be reduced to an `ite`. -/
1221-
@[simp] theorem dite_eq_ite : (dite P (fun _ ↦ a) fun _ ↦ b) = ite P a b := rfl
12221220
#align dite_eq_ite dite_eq_ite
12231221

12241222
theorem dite_eq_or_eq : (∃ h, dite P A B = A h) ∨ ∃ h, dite P A B = B h :=

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": "16d8352f7ed0d38cbc58ace03b3429d693cf50c6",
7+
"rev": "6b4cf96c89e53cfcd73350bbcd90333a051ff4f0",
88
"name": "std",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",

0 commit comments

Comments
 (0)