Skip to content

Commit 084c097

Browse files
committed
chore: use not_value at Nat.pow_pos
and remove `TODO` from `grind_lint_bitvec.lean`
1 parent 8afaa1b commit 084c097

File tree

2 files changed

+3
-4
lines changed

2 files changed

+3
-4
lines changed

src/Init/Data/Nat/Lemmas.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1095,6 +1095,7 @@ grind_pattern div_pow_of_pos => a ^ n where
10951095
guard n > 0
10961096

10971097
grind_pattern Nat.pow_pos => a ^ n where
1098+
not_value a -- Avoid excessive `BitVec` theorem instantiation (See `grind_lint_bitvec.lean`)
10981099
guard a > 0
10991100

11001101
protected theorem pow_add' (a m n : Nat) : a ^ (m + n) = a ^ n * a ^ m := by

tests/lean/run/grind_lint_bitvec.lean

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -7,13 +7,11 @@ import Lean.Elab.Tactic.Grind.LintExceptions
77
#guard_msgs in
88
#grind_lint inspect (min := 30) BitVec.msb_replicate
99

10-
-- TODO: Reduce limit after we add support for `no_value` constraint
1110
-- `BitVec.msb_signExtend` is reasonable at 22.
1211
#guard_msgs in
13-
#grind_lint inspect (min := 26) BitVec.msb_signExtend
12+
#grind_lint inspect (min := 22) BitVec.msb_signExtend
1413

1514
/-! Check BitVec namespace: -/
1615

17-
-- TODO: Reduce limit after we add support for `no_value` constraint. It was `20`
1816
#guard_msgs in
19-
#grind_lint check (min := 23) in BitVec
17+
#grind_lint check (min := 20) in BitVec

0 commit comments

Comments
 (0)