Skip to content

Commit 7289804

Browse files
authored
refactor: rename new option to debug.rawDecreasingByGoal (#5066)
as suggested by @semorrison in https://leanprover.zulipchat.com/#narrow/stream/116290-rss/topic/cleanDecreasingBy/near/462659021 Follow-up to #5016.
1 parent ca945be commit 7289804

File tree

2 files changed

+7
-7
lines changed

2 files changed

+7
-7
lines changed

src/Lean/Elab/PreDefinition/WF/Basic.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -9,17 +9,17 @@ import Lean.Elab.Tactic.Basic
99

1010
namespace Lean.Elab.WF
1111

12-
register_builtin_option cleanDecreasingByGoal : Bool := {
13-
defValue := true
14-
descr := "Cleans up internal implementation details in the proof goals presented by \
15-
`decreasing_by`, using the `clean_wf` tactic. Can be disabled for debugging \
16-
purposes. Please report an issue if you have to disable this option."
12+
register_builtin_option debug.rawDecreasingByGoal : Bool := {
13+
defValue := false
14+
descr := "Shows the raw `decreasing_by` goal including internal implementation detail \
15+
intead of cleaning it up with the `clean_wf` tactic. Can be enabled for debugging \
16+
purposes. Please report an issue if you have to use this option for other reasons."
1717
}
1818

1919
open Lean Elab Tactic
2020

2121
def applyCleanWfTactic : TacticM Unit := do
22-
if cleanDecreasingByGoal.get (← getOptions) then
22+
unless debug.rawDecreasingByGoal.get (← getOptions) do
2323
Tactic.evalTactic (← `(tactic| all_goals clean_wf))
2424

2525
end Lean.Elab.WF

tests/lean/run/4928.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -58,7 +58,7 @@ y : Nat
5858
(PSum.inr ⟨x.tail, y⟩) (PSum.inl ⟨x, y⟩)
5959
-/
6060
#guard_msgs in
61-
set_option cleanDecreasingByGoal false in
61+
set_option debug.rawDecreasingByGoal true in
6262
mutual
6363
def g1 (x : List Nat) (y : Nat) : Nat := g2 x.tail y
6464
termination_by x.length

0 commit comments

Comments
 (0)