Skip to content

Commit 366aa49

Browse files
committed
chore: bump std4 (#8548)
1 parent 81e04e3 commit 366aa49

File tree

5 files changed

+1
-18
lines changed

5 files changed

+1
-18
lines changed

Diff for: Mathlib/Data/List/Basic.lean

-7
Original file line numberDiff line numberDiff line change
@@ -642,13 +642,6 @@ theorem isEmpty_iff_eq_nil {l : List α} : l.isEmpty ↔ l = [] := by cases l <;
642642

643643
/-! ### dropLast -/
644644

645-
@[simp]
646-
theorem length_dropLast : ∀ l : List α, length l.dropLast = length l - 1
647-
| [] | [_] => rfl
648-
| a::b::l => by
649-
rw [dropLast, length_cons, length_cons, length_dropLast (b::l), succ_sub_one, length_cons,
650-
succ_sub_one]
651-
simp
652645
#align list.length_init List.length_dropLast
653646

654647
/-! ### getLast -/

Diff for: Mathlib/Data/Prod/Basic.lean

-3
Original file line numberDiff line numberDiff line change
@@ -125,9 +125,6 @@ theorem ext_iff {p q : α × β} : p = q ↔ p.1 = q.1 ∧ p.2 = q.2 := by
125125
rw [mk.inj_iff]
126126
#align prod.ext_iff Prod.ext_iff
127127

128-
@[ext]
129-
theorem ext {α β} {p q : α × β} (h₁ : p.1 = q.1) (h₂ : p.2 = q.2) : p = q :=
130-
ext_iff.2 ⟨h₁, h₂⟩
131128
#align prod.ext Prod.ext
132129

133130
theorem map_def {f : α → γ} {g : β → δ} : Prod.map f g = fun p : α × β ↦ (f p.1, g p.2) :=

Diff for: Mathlib/Data/Sigma/Basic.lean

-6
Original file line numberDiff line numberDiff line change
@@ -64,9 +64,6 @@ theorem eta : ∀ x : Σa, β a, Sigma.mk x.1 x.2 = x
6464
| ⟨_, _⟩ => rfl
6565
#align sigma.eta Sigma.eta
6666

67-
@[ext]
68-
theorem ext {x₀ x₁ : Sigma β} (h₀ : x₀.1 = x₁.1) (h₁ : HEq x₀.2 x₁.2) : x₀ = x₁ := by
69-
cases x₀; cases x₁; cases h₀; cases h₁; rfl
7067
#align sigma.ext Sigma.ext
7168

7269
theorem ext_iff {x₀ x₁ : Sigma β} : x₀ = x₁ ↔ x₀.1 = x₁.1 ∧ HEq x₀.2 x₁.2 := by
@@ -243,9 +240,6 @@ theorem mk.inj_iff {a₁ a₂ : α} {b₁ : β a₁} {b₂ : β a₂} :
243240
| _, _, _, _, Eq.refl _, HEq.refl _ => rfl
244241
#align psigma.mk.inj_iff PSigma.mk.inj_iff
245242

246-
@[ext]
247-
theorem ext {x₀ x₁ : PSigma β} (h₀ : x₀.1 = x₁.1) (h₁ : HEq x₀.2 x₁.2) : x₀ = x₁ := by
248-
cases x₀; cases x₁; cases h₀; cases h₁; rfl
249243
#align psigma.ext PSigma.ext
250244

251245
theorem ext_iff {x₀ x₁ : PSigma β} : x₀ = x₁ ↔ x₀.1 = x₁.1 ∧ HEq x₀.2 x₁.2 := by

Diff for: Mathlib/Logic/Basic.lean

-1
Original file line numberDiff line numberDiff line change
@@ -682,7 +682,6 @@ theorem exists_swap {p : α → β → Prop} : (∃ x y, p x y) ↔ ∃ y x, p x
682682
#align forall_exists_index forall_exists_index
683683

684684
#align exists_imp_distrib exists_imp
685-
alias ⟨_, not_exists_of_forall_not⟩ := exists_imp
686685
#align not_exists_of_forall_not not_exists_of_forall_not
687686

688687
#align Exists.some Exists.choose

Diff for: lake-manifest.json

+1-1
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": "a3b80114adc0948ff493f9acb6ee250f76922d80",
7+
"rev": "e403f680f0beb8610c29e6f799132e8be880554e",
88
"name": "std",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",

0 commit comments

Comments
 (0)