Skip to content

Commit

Permalink
merge nightly-testing
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Jan 4, 2025
2 parents 1a1a504 + c09b5d0 commit 42e5c0e
Show file tree
Hide file tree
Showing 5 changed files with 12 additions and 10 deletions.
4 changes: 2 additions & 2 deletions Aesop/RuleSet.lean
Original file line number Diff line number Diff line change
Expand Up @@ -372,7 +372,7 @@ def LocalRuleSet.erase (rs : LocalRuleSet) (f : RuleFilter) :
if let some decl := f.matchesSimpTheorem? then
for h : i in [:rs.simpTheoremsArray.size] do
have i_valid : i < simpTheoremsArray'.fst.size := by
simp_all [Membership.mem, simpTheoremsArray'.snd]
simp_all +zetaDelta [Membership.mem, simpTheoremsArray'.snd]
let (name, simpTheorems) := simpTheoremsArray'.fst[i]
if SimpTheorems.containsDecl simpTheorems decl then
let origin := .decl decl (inv := false)
Expand All @@ -383,7 +383,7 @@ def LocalRuleSet.erase (rs : LocalRuleSet) (f : RuleFilter) :
anyErased := true
let simpTheoremsArray := simpTheoremsArray'.fst
let simpTheoremsArrayNonempty : 0 < simpTheoremsArray.size := by
simp [simpTheoremsArray'.snd, rs.simpTheoremsArrayNonempty]
simp [simpTheoremsArray, simpTheoremsArray'.snd, rs.simpTheoremsArrayNonempty]
let rs := { rs with
localNormSimpRules, simpTheoremsArray, simpTheoremsArrayNonempty
}
Expand Down
4 changes: 3 additions & 1 deletion Aesop/Util/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -79,7 +79,9 @@ open DiscrTree

-- For `type = ∀ (x₁, ..., xₙ), T`, returns keys that match `T * ... *` (with
-- `n` stars).
def getConclusionDiscrTreeKeys (type : Expr) : MetaM (Array Key) :=

def getConclusionDiscrTreeKeys (type : Expr) :
MetaM (Array Key) :=
withoutModifyingState do
let (_, _, conclusion) ← forallMetaTelescope type
mkDiscrTreePath conclusion
Expand Down
2 changes: 1 addition & 1 deletion AesopTest/List.lean
Original file line number Diff line number Diff line change
Expand Up @@ -892,7 +892,7 @@ theorem last_append (l₁ l₂ : List α) (h : l₂ ≠ []) :
last (l₁ ++ l₂) (append_ne_nil_of_right_ne_nil l₁ h) = last l₂ h := by
induction l₁ <;> aesop

theorem last_concat {a : α} (l : List α) : last (concat l a) (concat_ne_nil a l) = a := by
theorem last_concat {a : α} (l : List α) : last (concat l a) (by exact X.concat_ne_nil a l) = a := by
aesop

@[simp] theorem last_singleton (a : α) : last [a] (cons_ne_nil a []) = a := rfl
Expand Down
2 changes: 1 addition & 1 deletion AesopTest/RulePattern.lean
Original file line number Diff line number Diff line change
Expand Up @@ -23,8 +23,8 @@ example (m n : Nat) : (↑m : Int) < 0 ∧ (↑n : Int) > 0 := by
set_option aesop.check.script false in
aesop!
all_goals
guard_hyp fwd_1 : 0 ≤ (m : Int)
guard_hyp fwd_2 : 0 ≤ (n : Int)
guard_hyp fwd_1 : 0 ≤ (m : Int)
falso

@[aesop safe forward (pattern := min x y)]
Expand Down
10 changes: 5 additions & 5 deletions AesopTest/SaturatePerformance.lean
Original file line number Diff line number Diff line change
Expand Up @@ -41,11 +41,11 @@ import Aesop
error: unsolved goals
α : Type u_1
l0 l1 l2 : List α
fwd : (l0 ++ l1).length ≥ 0
fwd_1 : (l0 ++ l1 ++ l2).length ≥ 0
fwd_2 : l2.length ≥ 0
fwd_3 : l0.length ≥ 0
fwd_4 : l1.length ≥ 0
fwd : l1.length ≥ 0
fwd_1 : (l0 ++ l1).length ≥ 0
fwd_2 : (l0 ++ l1 ++ l2).length ≥ 0
fwd_3 : l2.length ≥ 0
fwd_4 : l0.length ≥ 0
⊢ (l0 ++ l1 ++ l2).length = l0.length + l1.length + l2.length
-/
#guard_msgs in
Expand Down

0 comments on commit 42e5c0e

Please sign in to comment.