Skip to content

Commit

Permalink
chore: update RELEASES.md, add tests
Browse files Browse the repository at this point in the history
  • Loading branch information
collares committed Nov 1, 2023
1 parent 1f9a4f3 commit 41d9509
Show file tree
Hide file tree
Showing 2 changed files with 20 additions and 0 deletions.
2 changes: 2 additions & 0 deletions RELEASES.md
Original file line number Diff line number Diff line change
Expand Up @@ -11,6 +11,8 @@ of each version.
v4.4.0 (development in progress)
---------

* By default, `simp` will no longer try to use Decidable instances to rewrite terms. In particular, not all decidable goals will be closed by `simp`, and the `decide` tactic may be useful in such cases. The `decide` simp configuration option can be used to locally restore the old `simp` behavior, as in `simp (config := {decide := true})`; this includes using Decidable instances to verify side goals such as numeric inequalities.

v4.3.0
---------

Expand Down
18 changes: 18 additions & 0 deletions tests/lean/run/simpDecide.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,18 @@
example : 0 < 4 := by decide

example : 0 < 4 := by
fail_if_success { simp only }
simp (config := { decide := true }) only

def fib : Nat → Nat
| 0 => 0
| 1 => 1
| n+2 => fib (n+1) + fib n

theorem fib_two : fib 2 = 1 := rfl

example : 1 = fib (1 + 1) := by
fail_if_success { simp only [fib_two] }
simp (config := { decide := true }) only [fib_two]

example : 1 = fib (1 + 1) := by simp only [fib_two, (by decide : 1 + 1 = 2)]

0 comments on commit 41d9509

Please sign in to comment.