Skip to content

Commit

Permalink
second attempt to fix ci
Browse files Browse the repository at this point in the history
  • Loading branch information
luisacicolini committed Oct 3, 2024
1 parent e29e653 commit 12c2a38
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/Init/Data/BitVec/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1316,9 +1316,6 @@ theorem sshiftRight_msb_eq_msb {n : Nat} {x : BitVec w} :
intros h
simp [show n = 0 by omega]

@[deprecated sshiftRight_msb_eq_msb (since := "2024-10-03")]
abbrev msb_sshiftRight := @sshiftRight_msb_eq_msb

@[simp] theorem sshiftRight_zero {x : BitVec w} : x.sshiftRight 0 = x := by
ext i
simp [getLsbD_sshiftRight]
Expand Down Expand Up @@ -2943,4 +2940,7 @@ abbrev zeroExtend_truncate_succ_eq_zeroExtend_truncate_or_twoPow_of_getLsbD_true
@[deprecated and_one_eq_setWidth_ofBool_getLsbD (since := "2024-09-18")]
abbrev and_one_eq_zeroExtend_ofBool_getLsbD := @and_one_eq_setWidth_ofBool_getLsbD

@[deprecated sshiftRight_msb_eq_msb (since := "2024-10-03")]
abbrev msb_sshiftRight := @sshiftRight_msb_eq_msb

end BitVec

0 comments on commit 12c2a38

Please sign in to comment.