Skip to content

Commit e7a43ff

Browse files
committed
fix tests
1 parent 55bcda0 commit e7a43ff

File tree

3 files changed

+4
-4
lines changed

3 files changed

+4
-4
lines changed

src/Init/Core.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1371,7 +1371,7 @@ set_option linter.missingDocs false in
13711371
@[deprecated exists_of_subtype (since := "2025-04-04")]
13721372
abbrev existsOfSubtype := @exists_of_subtype
13731373

1374-
variable {α : Type u} {p : α → Prop}
1374+
variable {α : Sort u} {p : α → Prop}
13751375

13761376
protected theorem ext : ∀ {a1 a2 : {x // p x}}, val a1 = val a2 → a1 = a2
13771377
| ⟨_, _⟩, ⟨_, _⟩, rfl => rfl
@@ -1393,7 +1393,7 @@ instance {α : Type u} {p : α → Prop} [BEq α] [ReflBEq α] : ReflBEq {x : α
13931393
instance {α : Type u} {p : α → Prop} [BEq α] [LawfulBEq α] : LawfulBEq {x : α // p x} where
13941394
eq_of_beq h := Subtype.ext (eq_of_beq h)
13951395

1396-
instance {α : Type u} {p : α → Prop} [DecidableEq α] : DecidableEq {x : α // p x} :=
1396+
instance {α : Sort u} {p : α → Prop} [DecidableEq α] : DecidableEq {x : α // p x} :=
13971397
fun ⟨a, h₁⟩ ⟨b, h₂⟩ =>
13981398
if h : a = b then isTrue (by subst h; exact rfl)
13991399
else isFalse (fun h' => Subtype.noConfusion h' (fun h' => absurd h' h))

tests/lean/run/simp4.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -49,7 +49,7 @@ theorem ex8 (y x : Nat) : y = 0 → x + y = 0 → x = 0 := by
4949
simp (config := { contextual := true })
5050

5151
theorem ex9 (y x : Nat) : y = 0 → x + y = 0 → x = 0 := by
52-
fail_if_success simp [-Nat.add_eq_zero]
52+
fail_if_success simp [-Nat.add_eq_zero_iff]
5353
intro h₁ h₂
5454
simp [h₁] at h₂
5555
simp [h₂]

tests/lean/run/simpStar.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -20,7 +20,7 @@ h₂ : g x < 5
2020
-/
2121
#guard_msgs in
2222
theorem ex3 (x y : Nat) (h₁ : f x x = g x) (h₂ : f x x < 5) : f x x + f x x = 0 := by
23-
simp [*, -Nat.add_eq_zero] at *
23+
simp [*, -Nat.add_eq_zero_iff] at *
2424
trace_state
2525
have aux₁ : f x x = g x := h₁
2626
have aux₂ : g x < 5 := h₂

0 commit comments

Comments
 (0)