Skip to content

Commit 3fff2e2

Browse files
committed
rename two leftover instances
1 parent c7c566f commit 3fff2e2

File tree

1 file changed

+4
-4
lines changed

1 file changed

+4
-4
lines changed

src/Init/Data/BitVec/Lemmas.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -869,15 +869,15 @@ theorem append_def (x : BitVec v) (y : BitVec w) :
869869
(x ++ y).toNat = x.toNat <<< n ||| y.toNat :=
870870
rfl
871871

872-
@[simp] theorem getLsb_append {v : BitVec n} {w : BitVec m} :
873-
getLsb (v ++ w) i = bif i < m then getLsb w i else getLsb v (i - m) := by
872+
@[simp] theorem getLsb_append {x : BitVec n} {y : BitVec m} :
873+
getLsb (x ++ y) i = bif i < m then getLsb y i else getLsb x (i - m) := by
874874
simp only [append_def, getLsb_or, getLsb_shiftLeftZeroExtend, getLsb_zeroExtend']
875875
by_cases h : i < m
876876
· simp [h]
877877
· simp [h]; simp_all
878878

879-
@[simp] theorem getMsb_append {v : BitVec n} {w : BitVec m} :
880-
getMsb (v ++ w) i = bif n ≤ i then getMsb w (i - n) else getMsb v i := by
879+
@[simp] theorem getMsb_append {x : BitVec n} {y : BitVec m} :
880+
getMsb (x ++ y) i = bif n ≤ i then getMsb y (i - n) else getMsb x i := by
881881
simp [append_def]
882882
by_cases h : n ≤ i
883883
· simp [h]

0 commit comments

Comments
 (0)