Skip to content

Commit

Permalink
chore: bump toolchain to v4.3.0 (#87)
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em authored Nov 30, 2023
1 parent c7cff45 commit 76c4ea4
Show file tree
Hide file tree
Showing 7 changed files with 39 additions and 22 deletions.
11 changes: 9 additions & 2 deletions .gitignore
Original file line number Diff line number Diff line change
@@ -1,4 +1,11 @@
/build/
/tests/*.produced
/lake-packages

# macOS leaves these files everywhere:
.DS_Store
# Prior to v4.3.0-rc2 lake stored files in these locations.
# We'll leave them in the `.gitignore` for a while for users switching between toolchains.
/build/
/lake-packages/
/lakefile.olean
# After v4.3.0-rc2 lake stores its files here:
/.lake/
2 changes: 0 additions & 2 deletions AesopTest/Ext.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,5 @@ import Std.Tactic.Ext
example (f g : α → β) (h : ∀ a, f a = g a) : f = g := by
aesop

attribute [local ext] Prod

example (x y : α × β) (h₁ : x.1 = y.1) (h₂ : x.2 = y.2) : x = y := by
aesop
14 changes: 12 additions & 2 deletions AesopTest/HeartbeatLimit.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,17 +5,27 @@ Authors: Jannis Limperg
-/

import Aesop
import Std.Tactic.GuardMsgs

set_option aesop.check.all true
-- There is incorrectly a `linter.unreachableTactic` warning on
-- `aesop (options := { maxRuleHeartbeats := 1, terminal := true })`
-- below. This is perhaps because of a bad interaction with `#guard_msgs`?
set_option linter.unreachableTactic false

@[aesop safe constructors]
inductive Even : Nat → Prop
| zero : Even 0
| plusTwo : Even n → Even (n + 2)

/--
error: (deterministic) timeout at 'whnf', maximum number of heartbeats (1) has been reached (use 'set_option maxHeartbeats <num>' to set the limit)
-/
#guard_msgs in
example : Even 10 := by
aesop (options := { maxRuleHeartbeats := 1, terminal := true })

example : Even 10 := by
fail_if_success
aesop (options := { maxRuleHeartbeats := 1, terminal := true })
aesop

example (n m k : Nat) : n + m + k = (n + m) + k := by
Expand Down
6 changes: 3 additions & 3 deletions AesopTest/SeqCalcProver.lean
Original file line number Diff line number Diff line change
Expand Up @@ -273,14 +273,14 @@ abbrev Prove (φ : Form Φ) : Prop := Cal [] [] [] [φ]
example : Prove (⊥ ⇒ ♩0) := by simp
example : Prove (♩0 ⇒ ♩0) := by simp
example : Prove (♩0 ⇒ ♩1 ⇒ ♩0) := by simp
example : ¬ Prove (♩0 ⇒ ♩1) := by simp
example : ¬ Prove (♩0 ⇒ ♩1) := by simp (config := {decide := true})


--- Soundness and Completeness

@[simp]
def SC' (i : Φ → Prop) (l r : List Φ) (Γ Δ : List (Form Φ)) : Prop :=
SC i (Γ ++ l.map (♩·)) (Δ ++ r.map (♩·))
SC i (Γ ++ l.map (♩·)) (Δ ++ r.map (♩·))

theorem Cal_sound_complete [DecidableEq Φ]
(l r : List Φ) (Γ Δ : List (Form Φ))
Expand Down Expand Up @@ -439,7 +439,7 @@ end Proof

@[simp]
def Proof' (l r : List Φ) (Γ Δ : List (Form Φ)) : Prop :=
Proof (Γ ++ l.map (♩·)) (Δ ++ r.map (♩·))
Proof (Γ ++ l.map (♩·)) (Δ ++ r.map (♩·))

theorem Cal_Proof [DecidableEq Φ]
(l r : List Φ) (Γ Δ : List (Form Φ)) (h : Cal l r Γ Δ)
Expand Down
24 changes: 13 additions & 11 deletions lake-manifest.json
Original file line number Diff line number Diff line change
@@ -1,12 +1,14 @@
{"version": 6,
"packagesDir": "lake-packages",
{"version": 7,
"packagesDir": ".lake/packages",
"packages":
[{"git":
{"url": "https://github.com/leanprover/std4",
"subDir?": null,
"rev": "9bfbd2a12ee9cf2e159a8a6b4d1ef6c149728f66",
"opts": {},
"name": "std",
"inputRev?": "main",
"inherited": false}}],
"name": "aesop"}
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "2e4a3586a8f16713f16b2d2b3af3d8e65f3af087",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inherited": false,
"configFile": "lakefile.lean"}],
"name": "aesop",
"lakeDir": ".lake"}
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.3.0-rc1
leanprover/lean4:v4.3.0
2 changes: 1 addition & 1 deletion tests/TraceProof.lean.expected
Original file line number Diff line number Diff line change
Expand Up @@ -4,4 +4,4 @@ tests/TraceProof.lean:14:2: error: tactic 'aesop' failed, made no progress
tests/TraceProof.lean:20:2: warning: aesop: failed to prove the goal after exhaustive search.
tests/TraceProof.lean:19:15: error: unsolved goals
⊢ False
[aesop.proof] id ?m.38
[aesop.proof] id ?m.36

0 comments on commit 76c4ea4

Please sign in to comment.