Skip to content

Commit

Permalink
chore: the previous commit exposed an issue with simp
Browse files Browse the repository at this point in the history
`simp` was previously swallowing runtime exceptions and masking an
issue with this example.

`runT` is defined by well-founded recursion, but reducing the ground
term `runT x` takes a long time when `decide := true`.

Remark PR #2722 changes the `decide` default value to `false`.

When `decide := true`, we should probably have better diagnostics /
error messages for this kind of situation.
  • Loading branch information
leodemoura committed Nov 3, 2023
1 parent 4afcdeb commit 47c09ac
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion tests/lean/run/lazyUnfoldingPerfIssue.lean
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,7 @@ theorem equivalent: Run.run x = Run.run x := by
apply Eq.refl (runT x)

example : Run.run x = Run.run x := by
simp [Run.run]
simp (config := { decide := false }) [Run.run]

end Ex1

Expand Down

0 comments on commit 47c09ac

Please sign in to comment.