Skip to content

Commit eda0afd

Browse files
committed
merge lean-pr-testing-10204
2 parents 4f16e03 + 033343f commit eda0afd

File tree

5 files changed

+3
-7
lines changed

5 files changed

+3
-7
lines changed

Aesop/Check.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -16,8 +16,7 @@ namespace Aesop
1616
initialize Check.all : Lean.Option Bool ←
1717
Option.register `aesop.check.all
1818
{ defValue := false
19-
descr := "(aesop) Enable all runtime checks. Individual checks can still be disabled."
20-
group := "tactic" }
19+
descr := "(aesop) Enable all runtime checks. Individual checks can still be disabled." }
2120

2221
structure Check where
2322
toOption : Lean.Option Bool
@@ -42,7 +41,7 @@ end Check
4241
local macro "register_aesop_check_option" optName:ident descr:str : command =>
4342
`(initialize option : Lean.Option Bool ←
4443
Lean.Option.register $(quote $ `aesop.check ++ optName.getId)
45-
{ defValue := false, descr := $descr, group := "tactic" }
44+
{ defValue := false, descr := $descr }
4645

4746
def $(mkIdent $ `Check ++ optName.getId) : Aesop.Check := ⟨option⟩)
4847

Aesop/Stats/Basic.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -18,7 +18,6 @@ namespace Aesop
1818
initialize collectStatsOption : Lean.Option Bool ←
1919
Lean.Option.register `aesop.collectStats {
2020
defValue := false
21-
group := "aesop"
2221
descr := "(aesop) collect statistics about Aesop invocations. Use #aesop_stats to display the collected statistics."
2322
}
2423

Aesop/Tracing.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -25,7 +25,6 @@ def registerTraceOption (traceName : Name) (descr : String) :
2525
IO TraceOption := do
2626
let option ← Option.register (`trace.aesop ++ traceName) {
2727
defValue := false
28-
group := "trace"
2928
descr
3029
}
3130
return { traceClass := `aesop ++ traceName, option }

Aesop/Util/Basic.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -445,7 +445,6 @@ def elabPattern (stx : Syntax) : TermElabM Expr :=
445445

446446
register_option aesop.smallErrorMessages : Bool := {
447447
defValue := false
448-
group := "aesop"
449448
descr := "(aesop) Print smaller error messages. Used for testing."
450449
}
451450

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4-pr-releases:pr-release-10204-faccc35
1+
leanprover/lean4:nightly-2025-11-27

0 commit comments

Comments
 (0)