Skip to content

Commit ba9a63b

Browse files
authored
chore: bump toolchain to v4.17.0-rc1 (#195)
1 parent 44dab9f commit ba9a63b

File tree

5 files changed

+9
-10
lines changed

5 files changed

+9
-10
lines changed

AesopTest/List.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -540,7 +540,6 @@ theorem X.append_ne_nil_of_ne_nil_left (s t : List α) : s ≠ [] → s ++ t ≠
540540
theorem X.append_ne_nil_of_ne_nil_right (s t : List α) : t ≠ [] → s ++ t ≠ [] := by
541541
induction s <;> aesop
542542

543-
attribute [-simp] append_eq_nil
544543
@[simp] theorem X.append_eq_nil {p q : List α} : (p ++ q) = [] ↔ p = [] ∧ q = [] := by
545544
aesop (add 1% cases List)
546545

@@ -718,7 +717,7 @@ theorem replicate_right_injective (a : α) : Injective (λ n => replicate n a) :
718717
/-! ### flatMap -/
719718

720719
instance : Bind List where
721-
bind l f := List.flatMap l f
720+
bind l f := List.flatMap f l
722721

723722
@[simp] theorem bind_eq_flatMap {α β} (f : α → List β) (l : List α) :
724723
l >>= f = l.flatMap f := rfl

AesopTest/RulePattern.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -23,8 +23,8 @@ example (m n : Nat) : (↑m : Int) < 0 ∧ (↑n : Int) > 0 := by
2323
set_option aesop.check.script false in
2424
aesop!
2525
all_goals
26-
guard_hyp fwd_2 : 0 ≤ (n : Int)
27-
guard_hyp fwd_1 : 0 ≤ (m : Int)
26+
guard_hyp fwd : 0 ≤ (n : Int)
27+
guard_hyp fwd_2 : 0 ≤ (m : Int)
2828
falso
2929

3030
@[aesop safe forward (pattern := min x y)]
@@ -44,8 +44,8 @@ axiom triangle (a b : Int) : |a + b| ≤ |a| + |b|
4444

4545
example : |a + b| ≤ |c + d| := by
4646
aesop!
47-
guard_hyp fwd : |c + d| ≤ |c| + |d|
48-
guard_hyp fwd_1 : |a + b| ≤ |a| + |b|
47+
guard_hyp fwd_1 : |c + d| ≤ |c| + |d|
48+
guard_hyp fwd : |a + b| ≤ |a| + |b|
4949
falso
5050

5151
@[aesop safe apply (pattern := (0 : Nat))]

lake-manifest.json

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -5,10 +5,10 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "01006c9e86bf9e397c026fef4190478dd1fd897e",
8+
"rev": "512d7fa38234139a34c04e3b3438fc142b51bbee",
99
"name": "batteries",
1010
"manifestFile": "lake-manifest.json",
11-
"inputRev": "v4.16.0",
11+
"inputRev": "v4.17.0-rc1",
1212
"inherited": false,
1313
"configFile": "lakefile.toml"}],
1414
"name": "aesop",

lakefile.toml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ precompileModules = false # We would like to turn this on, but it breaks the Mat
66
[[require]]
77
name = "batteries"
88
git = "https://github.com/leanprover-community/batteries"
9-
rev = "v4.16.0"
9+
rev = "v4.17.0-rc1"
1010

1111
[[lean_lib]]
1212
name = "Aesop"

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.16.0
1+
leanprover/lean4:v4.17.0-rc1

0 commit comments

Comments
 (0)