File tree Expand file tree Collapse file tree 2 files changed +7
-7
lines changed
src/Lean/Elab/PreDefinition/WF Expand file tree Collapse file tree 2 files changed +7
-7
lines changed Original file line number Diff line number Diff line change @@ -9,17 +9,17 @@ import Lean.Elab.Tactic.Basic
9
9
10
10
namespace Lean.Elab.WF
11
11
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 ."
17
17
}
18
18
19
19
open Lean Elab Tactic
20
20
21
21
def applyCleanWfTactic : TacticM Unit := do
22
- if cleanDecreasingByGoal. get (← getOptions) then
22
+ unless debug.rawDecreasingByGoal. get (← getOptions) do
23
23
Tactic.evalTactic (← `(tactic| all_goals clean_wf))
24
24
25
25
end Lean.Elab.WF
Original file line number Diff line number Diff line change @@ -58,7 +58,7 @@ y : Nat
58
58
(PSum.inr ⟨x.tail, y⟩) (PSum.inl ⟨x, y⟩)
59
59
-/
60
60
#guard_msgs in
61
- set_option cleanDecreasingByGoal false in
61
+ set_option debug.rawDecreasingByGoal true in
62
62
mutual
63
63
def g1 (x : List Nat) (y : Nat) : Nat := g2 x.tail y
64
64
termination_by x.length
You can’t perform that action at this time.
0 commit comments