Skip to content

Commit

Permalink
Bump to nightly-2023-08-17
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em authored and JLimperg committed Aug 17, 2023
1 parent 147e0c7 commit 0607eb4
Show file tree
Hide file tree
Showing 3 changed files with 8 additions and 4 deletions.
2 changes: 2 additions & 0 deletions AesopTest/List.lean
Original file line number Diff line number Diff line change
Expand Up @@ -89,6 +89,7 @@ instance : Membership α (Option α) :=

@[simp]
theorem mem_spec {o : Option α} : a ∈ o ↔ o = some a := by
set_option aesop.check.script false in -- TODO
aesop (add norm simp Membership.mem)

@[simp]
Expand Down Expand Up @@ -305,6 +306,7 @@ theorem mem_map_of_injective {f : α → β} (H : Injective f) {a : α} {l : Lis
@[simp] theorem _root_.function.involutive.exists_mem_and_apply_eq_iff {f : α → α}
(hf : Involutive f) (x : α) (l : List α) :
(∃ (y : α), y ∈ l ∧ f y = x) ↔ f x ∈ l := by
set_option aesop.check.script false in -- TODO
aesop

theorem mem_map_of_involutive {f : α → α} (hf : Involutive f) {a : α} {l : List α} :
Expand Down
8 changes: 5 additions & 3 deletions lake-manifest.json
Original file line number Diff line number Diff line change
@@ -1,9 +1,11 @@
{"version": 4,
{"version": 5,
"packagesDir": "lake-packages",
"packages":
[{"git":
{"url": "https://github.com/leanprover/std4",
"subDir?": null,
"rev": "dbffa8cb31b0c51b151453c4ff8f00ede2a84ed8",
"rev": "49353fa54abdac7221fe27f7b57a6ed9ff559d5c",
"opts": {},
"name": "std",
"inputRev?": "main"}}]}
"inputRev?": "main",
"inherited": false}}]}
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:nightly-2023-07-29
leanprover/lean4:nightly-2023-08-17

0 comments on commit 0607eb4

Please sign in to comment.