Skip to content

Commit 4bcbef8

Browse files
committed
fix tests
1 parent 6c3a6bf commit 4bcbef8

File tree

3 files changed

+8
-8
lines changed

3 files changed

+8
-8
lines changed

tests/lean/run/4313.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ theorem bmod_add_bmod_congr : Int.bmod (Int.bmod x n + y) n = Int.bmod (x + y) n
2121
rw [bmod_def x n]
2222
split -- `split` now generates the more meaningful `isTrue` and `isFalse` tags.
2323
case isTrue p =>
24-
simp only [emod_add_bmod_congr]
24+
simp only [emod_add_bmod]
2525
case isFalse p =>
2626
rw [Int.sub_eq_add_neg, Int.add_right_comm, ←Int.sub_eq_add_neg]
2727
simp

tests/lean/run/partial_fixpoint_induct.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -183,7 +183,7 @@ theorem List.findIndex_implies_pred (xs : List α) (p : α → Bool) :
183183
have : r = 0 := by simp_all
184184
simp_all
185185
next =>
186-
simp only [Option.map_eq_map, Option.map_eq_some'] at hsome
186+
simp only [Option.map_eq_map, Option.map_eq_some_iff] at hsome
187187
obtain ⟨r', hr, rfl⟩ := hsome
188188
specialize ih _ _ hr
189189
simpa

tests/lean/run/simpConfigPropagationIssue1.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -2,12 +2,12 @@ namespace Option
22

33
variable {α : Type _}
44

5-
instance liftOrGet_isCommutative (f : α → α → α) [Std.Commutative f] :
6-
Std.Commutative (liftOrGet f) :=
7-
⟨fun a b ↦ by cases a <;> cases b <;> simp [liftOrGet, Std.Commutative.comm]⟩
5+
instance merge_isCommutative (f : α → α → α) [Std.Commutative f] :
6+
Std.Commutative (merge f) :=
7+
⟨fun a b ↦ by cases a <;> cases b <;> simp [merge, Std.Commutative.comm]⟩
88

9-
instance liftOrGet_isAssociative (f : α → α → α) [Std.Associative f] :
10-
Std.Associative (liftOrGet f) :=
11-
⟨fun a b c ↦ by cases a <;> cases b <;> cases c <;> simp [liftOrGet, Std.Associative.assoc]⟩
9+
instance merge_isAssociative (f : α → α → α) [Std.Associative f] :
10+
Std.Associative (merge f) :=
11+
⟨fun a b c ↦ by cases a <;> cases b <;> cases c <;> simp [merge, Std.Associative.assoc]⟩
1212

1313
end Option

0 commit comments

Comments
 (0)