Skip to content

Commit 86ecbac

Browse files
committed
chore: bump Std (leanprover-community#10177)
There's an exciting linter failure on `bump/v4.6.0`, and I'm wondering if this is caused by strange simp lemmas in leanprover-community/batteries#558, so I'm updating to that before the bump. Co-authored-by: Scott Morrison <[email protected]>
1 parent e7d0ec3 commit 86ecbac

File tree

4 files changed

+1
-9
lines changed

4 files changed

+1
-9
lines changed

Mathlib/Data/BitVec/Lemmas.lean

Lines changed: 0 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -70,8 +70,6 @@ theorem addLsb_eq_twice_add_one {x b} : addLsb x b = 2 * x + cond b 1 0 := by
7070
-- Since the statement is awkward and `Std.BitVec` has no comparable API, we just drop it.
7171
#noalign bitvec.to_nat_eq_foldr_reverse
7272

73-
theorem toNat_lt {n : ℕ} (v : BitVec n) : v.toNat < 2 ^ n := by
74-
exact v.toFin.2
7573
#align bitvec.to_nat_lt Std.BitVec.toNat_lt
7674

7775
theorem addLsb_div_two {x b} : addLsb x b / 2 = x := by
@@ -132,8 +130,6 @@ variable (x y : Fin (2^w))
132130
simp only [HXor.hXor, Xor.xor, Fin.xor, BitVec.xor, toNat_ofFin, ofFin.injEq, Fin.mk.injEq]
133131
exact mod_eq_of_lt (Nat.xor_lt_two_pow x.prop y.prop)
134132

135-
@[simp] lemma ofFin_add : ofFin (x + y) = ofFin x + ofFin y := rfl
136-
@[simp] lemma ofFin_sub : ofFin (x - y) = ofFin x - ofFin y := rfl
137133
@[simp] lemma ofFin_mul : ofFin (x * y) = ofFin x * ofFin y := rfl
138134

139135
-- These should be simp, but Std's simp-lemmas do not allow this yet.

Mathlib/Data/Fin/Basic.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -209,8 +209,6 @@ section Order
209209
#align fin.is_le Fin.is_le
210210
#align fin.is_le' Fin.is_le'
211211

212-
theorem lt_iff_val_lt_val {a b : Fin n} : a < b ↔ (a : ℕ) < b :=
213-
Iff.rfl
214212
#align fin.lt_iff_coe_lt_coe Fin.lt_iff_val_lt_val
215213

216214
theorem le_iff_val_le_val {a b : Fin n} : a ≤ b ↔ (a : ℕ) ≤ b :=

Mathlib/Data/Nat/Bitwise.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -129,12 +129,10 @@ theorem xor_bit : ∀ a m b n, bit a m ^^^ bit b n = bit (bne a b) (m ^^^ n) :=
129129
attribute [simp] Nat.testBit_bitwise
130130
#align nat.test_bit_bitwise Nat.testBit_bitwise
131131

132-
@[simp]
133132
theorem testBit_lor : ∀ m n k, testBit (m ||| n) k = (testBit m k || testBit n k) :=
134133
testBit_bitwise rfl
135134
#align nat.test_bit_lor Nat.testBit_lor
136135

137-
@[simp]
138136
theorem testBit_land : ∀ m n k, testBit (m &&& n) k = (testBit m k && testBit n k) :=
139137
testBit_bitwise rfl
140138
#align nat.test_bit_land Nat.testBit_land

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@
44
[{"url": "https://github.com/leanprover/std4",
55
"type": "git",
66
"subDir": null,
7-
"rev": "08ec2584b1892869e3a5f4122b029989bcb4ca79",
7+
"rev": "bdec3daab8481a5750e255c9bdf8bf087370908b",
88
"name": "std",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",

0 commit comments

Comments
 (0)