You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
In the following example, aesop does not terminate (for at least 20 minutes). Besides my hope that aesop might actually solve the goal, is "running forever" an intended behavior? This is the first time I've seen where it doesn't quickly run out of "iterations" or heartbeats or something.
The example arose while making a differentiability tactic, like Mathlib's current continuity. For reproducing the issue, cheking out the Mathlib PR may be convenient.
import Mathlib.Data.Complex.Exponential
open Real (cos)
axiomMyDifferentiable : (ℝ → ℝ) → PropaxiomMyDifferentiable.cos {f : ℝ → ℝ} :
MyDifferentiable f → MyDifferentiable fun x => cos (f x)
example : MyDifferentiable fun y ↦ (Complex.cosh ↑(cos y)).re := by
aesop (add safe MyDifferentiable.cos) (rule_sets [-builtin,-default])
apply MyDifferentiable.cos in the same place runs out of heartbeats, so that may have something to do with it. But I haven't yet figured out why Aesop doesn't run out of heartbeats as well.
In the following example,
aesop
does not terminate (for at least 20 minutes). Besides my hope that aesop might actually solve the goal, is "running forever" an intended behavior? This is the first time I've seen where it doesn't quickly run out of "iterations" or heartbeats or something.The example arose while making a
differentiability
tactic, like Mathlib's currentcontinuity
. For reproducing the issue, cheking out the Mathlib PR may be convenient.The text was updated successfully, but these errors were encountered: