Skip to content

Commit

Permalink
chore: fix docstrings
Browse files Browse the repository at this point in the history
  • Loading branch information
luisacicolini committed Jan 14, 2025
1 parent 8c64c87 commit 8c3448f
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/Init/Data/BitVec/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -676,28 +676,28 @@ def ofBoolListLE : (bs : List Bool) → BitVec bs.length

def not_overflow {w : Nat} (x : BitVec w) : Bool := x.toInt == - (2 ^ (w - 1))

/-- Overflow predicate for unsigned addition modulo 2^m.
/-- Overflow predicate for unsigned addition modulo 2^w.
SMT-Lib name: `bvuaddo`.
-/

def uadd_overflow {w : Nat} (x y : BitVec w) : Bool := x.toNat + y.toNat ≥ 2 ^ w

/-- Overflow predicate for signed addition on m-bit 2's complement.
/-- Overflow predicate for signed addition on w-bit 2's complement.
SMT-Lib name: `bvsaddo`.
-/

def sadd_overflow {w : Nat} (x y : BitVec w) : Bool := (x.toInt + y.toInt ≥ 2 ^ (w - 1)) || (x.toInt + y.toInt < - 2 ^ (w - 1))

/-- Overflow predicate for unsigned multiplication modulo 2^m.
/-- Overflow predicate for unsigned multiplication modulo 2^w.
SMT-Lib name: `bvumulo`.
-/

def umul_overflow {w : Nat} (x y : BitVec w) : Bool := x.toNat * y.toNat ≥ 2 ^ w

/-- Overflow predicate for signed multiplication on m-bit 2's complement.
/-- Overflow predicate for signed multiplication on w-bit 2's complement.
SMT-Lib name: `bvsmulo`.
-/
Expand Down

0 comments on commit 8c3448f

Please sign in to comment.