Skip to content

Commit b8eba16

Browse files
committed
feat: revert "feat: disable "experimental" warning for mvcgen (#10638)"
This reverts commit 689b3aa.
1 parent 54c6efe commit b8eba16

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

src/Lean/Elab/Tactic/Do/VCGen.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -448,7 +448,7 @@ where
448448
@[builtin_tactic Lean.Parser.Tactic.mvcgen]
449449
def elabMVCGen : Tactic := fun stx => withMainContext do
450450
if mvcgen.warning.get (← getOptions) then
451-
logWarningAt stx "The `mvcgen` tactic is new and its behavior may change in the future. This project has used `set_option mvcgen.warning true` to discourage its use."
451+
logWarningAt stx "The `mvcgen` tactic is experimental and still under development. Avoid using it in production projects."
452452
let ctx ← mkSpecContext stx[1] stx[2]
453453
let fuel := match ctx.config.stepLimit with
454454
| some n => .limited n

src/Lean/Elab/Tactic/Do/VCGen/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -18,9 +18,9 @@ open Lean Parser Elab Tactic Meta Do SpecAttr
1818
builtin_initialize registerTraceClass `Elab.Tactic.Do.vcgen
1919

2020
register_builtin_option mvcgen.warning : Bool := {
21-
defValue := false
21+
defValue := true
2222
group := "debug"
23-
descr := "enable `mvcgen` usage warning"
23+
descr := "disable `mvcgen` usage warning"
2424
}
2525

2626
inductive Fuel where

0 commit comments

Comments
 (0)