File tree Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -2026,9 +2026,9 @@ theorem sub_def {n} (x y : BitVec n) : x - y = .ofNat n ((2^n - y.toNat) + x.toN
2026
2026
2027
2027
@[simp] theorem toFin_sub (x y : BitVec n) : (x - y).toFin = toFin x - toFin y := rfl
2028
2028
2029
- @[simp] theorem ofFin_sub (x : Fin (2 ^n)) (y : BitVec n) : .ofFin x - y = .ofFin (x - y.toFin) :=
2029
+ theorem ofFin_sub (x : Fin (2 ^n)) (y : BitVec n) : .ofFin x - y = .ofFin (x - y.toFin) :=
2030
2030
rfl
2031
- @[simp] theorem sub_ofFin (x : BitVec n) (y : Fin (2 ^n)) : x - .ofFin y = .ofFin (x.toFin - y) :=
2031
+ theorem sub_ofFin (x : BitVec n) (y : Fin (2 ^n)) : x - .ofFin y = .ofFin (x.toFin - y) :=
2032
2032
rfl
2033
2033
2034
2034
-- Remark: we don't use `[simp]` here because simproc` subsumes it for literals.
You can’t perform that action at this time.
0 commit comments