Equations
- One or more equations did not get rendered due to their size.
Instances For
theorem
UInt8.toNat_shiftRight
(a b : UInt8)
:
Eq (HShiftRight.hShiftRight a b).toNat (HShiftRight.hShiftRight a.toNat (HMod.hMod b.toNat 8))
theorem
UInt8.toNat_shiftLeft
(a b : UInt8)
:
Eq (HShiftLeft.hShiftLeft a b).toNat (HMod.hMod (HShiftLeft.hShiftLeft a.toNat (HMod.hMod b.toNat 8)) (HPow.hPow 2 8))
theorem
UInt8.toBitVec_shiftRight
(a b : UInt8)
:
Eq (HShiftRight.hShiftRight a b).toBitVec (HShiftRight.hShiftRight a.toBitVec (HMod.hMod b.toBitVec 8))
theorem
UInt8.toBitVec_shiftLeft
(a b : UInt8)
:
Eq (HShiftLeft.hShiftLeft a b).toBitVec (HShiftLeft.hShiftLeft a.toBitVec (HMod.hMod b.toBitVec 8))
theorem
UInt16.toNat_shiftRight
(a b : UInt16)
:
Eq (HShiftRight.hShiftRight a b).toNat (HShiftRight.hShiftRight a.toNat (HMod.hMod b.toNat 16))
theorem
UInt16.toBitVec_shiftLeft
(a b : UInt16)
:
Eq (HShiftLeft.hShiftLeft a b).toBitVec (HShiftLeft.hShiftLeft a.toBitVec (HMod.hMod b.toBitVec 16))
theorem
UInt16.toBitVec_shiftRight
(a b : UInt16)
:
Eq (HShiftRight.hShiftRight a b).toBitVec (HShiftRight.hShiftRight a.toBitVec (HMod.hMod b.toBitVec 16))
theorem
UInt16.toNat_shiftLeft
(a b : UInt16)
:
Eq (HShiftLeft.hShiftLeft a b).toNat (HMod.hMod (HShiftLeft.hShiftLeft a.toNat (HMod.hMod b.toNat 16)) (HPow.hPow 2 16))
theorem
UInt32.toNat_shiftLeft
(a b : UInt32)
:
Eq (HShiftLeft.hShiftLeft a b).toNat (HMod.hMod (HShiftLeft.hShiftLeft a.toNat (HMod.hMod b.toNat 32)) (HPow.hPow 2 32))
theorem
UInt32.toBitVec_shiftRight
(a b : UInt32)
:
Eq (HShiftRight.hShiftRight a b).toBitVec (HShiftRight.hShiftRight a.toBitVec (HMod.hMod b.toBitVec 32))
theorem
UInt32.toBitVec_shiftLeft
(a b : UInt32)
:
Eq (HShiftLeft.hShiftLeft a b).toBitVec (HShiftLeft.hShiftLeft a.toBitVec (HMod.hMod b.toBitVec 32))
theorem
UInt32.toNat_shiftRight
(a b : UInt32)
:
Eq (HShiftRight.hShiftRight a b).toNat (HShiftRight.hShiftRight a.toNat (HMod.hMod b.toNat 32))
theorem
UInt64.toBitVec_shiftLeft
(a b : UInt64)
:
Eq (HShiftLeft.hShiftLeft a b).toBitVec (HShiftLeft.hShiftLeft a.toBitVec (HMod.hMod b.toBitVec 64))
theorem
UInt64.toBitVec_shiftRight
(a b : UInt64)
:
Eq (HShiftRight.hShiftRight a b).toBitVec (HShiftRight.hShiftRight a.toBitVec (HMod.hMod b.toBitVec 64))
theorem
UInt64.toNat_shiftRight
(a b : UInt64)
:
Eq (HShiftRight.hShiftRight a b).toNat (HShiftRight.hShiftRight a.toNat (HMod.hMod b.toNat 64))
theorem
UInt64.toNat_shiftLeft
(a b : UInt64)
:
Eq (HShiftLeft.hShiftLeft a b).toNat (HMod.hMod (HShiftLeft.hShiftLeft a.toNat (HMod.hMod b.toNat 64)) (HPow.hPow 2 64))
theorem
Bool.toBitVec_toUInt8
{b : Bool}
:
Eq b.toUInt8.toBitVec (BitVec.setWidth 8 (BitVec.ofBool b))
theorem
Bool.toBitVec_toUInt16
{b : Bool}
:
Eq b.toUInt16.toBitVec (BitVec.setWidth 16 (BitVec.ofBool b))
theorem
Bool.toBitVec_toUInt32
{b : Bool}
:
Eq b.toUInt32.toBitVec (BitVec.setWidth 32 (BitVec.ofBool b))
theorem
Bool.toBitVec_toUInt64
{b : Bool}
:
Eq b.toUInt64.toBitVec (BitVec.setWidth 64 (BitVec.ofBool b))
theorem
UInt8.toUInt16_not
(a : UInt8)
:
Eq (Complement.complement a).toUInt16 (HMod.hMod (Complement.complement a.toUInt16) 256)
theorem
UInt8.toUInt32_not
(a : UInt8)
:
Eq (Complement.complement a).toUInt32 (HMod.hMod (Complement.complement a.toUInt32) 256)
theorem
UInt8.toUInt64_not
(a : UInt8)
:
Eq (Complement.complement a).toUInt64 (HMod.hMod (Complement.complement a.toUInt64) 256)
theorem
UInt8.toUSize_not
(a : UInt8)
:
Eq (Complement.complement a).toUSize (HMod.hMod (Complement.complement a.toUSize) 256)
theorem
UInt16.toUInt32_not
(a : UInt16)
:
Eq (Complement.complement a).toUInt32 (HMod.hMod (Complement.complement a.toUInt32) 65536)
theorem
UInt16.toUInt64_not
(a : UInt16)
:
Eq (Complement.complement a).toUInt64 (HMod.hMod (Complement.complement a.toUInt64) 65536)
theorem
UInt16.toUSize_not
(a : UInt16)
:
Eq (Complement.complement a).toUSize (HMod.hMod (Complement.complement a.toUSize) 65536)
theorem
UInt32.toUInt64_not
(a : UInt32)
:
Eq (Complement.complement a).toUInt64 (HMod.hMod (Complement.complement a.toUInt64) 4294967296)
theorem
UInt32.toUSize_not
(a : UInt32)
:
Eq (Complement.complement a).toUSize (HMod.hMod (Complement.complement a.toUSize) 4294967296)
theorem
UInt8.toFin_shiftLeft
(a b : UInt8)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toFin (HShiftLeft.hShiftLeft a.toFin b.toFin)
theorem
UInt16.toFin_shiftLeft
(a b : UInt16)
(hb : LT.lt b 16)
:
Eq (HShiftLeft.hShiftLeft a b).toFin (HShiftLeft.hShiftLeft a.toFin b.toFin)
theorem
UInt32.toFin_shiftLeft
(a b : UInt32)
(hb : LT.lt b 32)
:
Eq (HShiftLeft.hShiftLeft a b).toFin (HShiftLeft.hShiftLeft a.toFin b.toFin)
theorem
UInt64.toFin_shiftLeft
(a b : UInt64)
(hb : LT.lt b 64)
:
Eq (HShiftLeft.hShiftLeft a b).toFin (HShiftLeft.hShiftLeft a.toFin b.toFin)
theorem
USize.toFin_shiftLeft
(a b : USize)
(hb : LT.lt b.toNat System.Platform.numBits)
:
Eq (HShiftLeft.hShiftLeft a b).toFin (HShiftLeft.hShiftLeft a.toFin b.toFin)
theorem
UInt8.shiftLeft_eq_shiftLeft_mod
(a b : UInt8)
:
Eq (HShiftLeft.hShiftLeft a b) (HShiftLeft.hShiftLeft a (HMod.hMod b 8))
theorem
UInt16.shiftLeft_eq_shiftLeft_mod
(a b : UInt16)
:
Eq (HShiftLeft.hShiftLeft a b) (HShiftLeft.hShiftLeft a (HMod.hMod b 16))
theorem
UInt32.shiftLeft_eq_shiftLeft_mod
(a b : UInt32)
:
Eq (HShiftLeft.hShiftLeft a b) (HShiftLeft.hShiftLeft a (HMod.hMod b 32))
theorem
UInt64.shiftLeft_eq_shiftLeft_mod
(a b : UInt64)
:
Eq (HShiftLeft.hShiftLeft a b) (HShiftLeft.hShiftLeft a (HMod.hMod b 64))
theorem
USize.shiftLeft_eq_shiftLeft_mod
(a b : USize)
:
Eq (HShiftLeft.hShiftLeft a b) (HShiftLeft.hShiftLeft a (HMod.hMod b (ofNat System.Platform.numBits)))
theorem
UInt8.shiftRight_eq_shiftRight_mod
(a b : UInt8)
:
Eq (HShiftRight.hShiftRight a b) (HShiftRight.hShiftRight a (HMod.hMod b 8))
theorem
UInt16.shiftRight_eq_shiftRight_mod
(a b : UInt16)
:
Eq (HShiftRight.hShiftRight a b) (HShiftRight.hShiftRight a (HMod.hMod b 16))
theorem
UInt32.shiftRight_eq_shiftRight_mod
(a b : UInt32)
:
Eq (HShiftRight.hShiftRight a b) (HShiftRight.hShiftRight a (HMod.hMod b 32))
theorem
UInt64.shiftRight_eq_shiftRight_mod
(a b : UInt64)
:
Eq (HShiftRight.hShiftRight a b) (HShiftRight.hShiftRight a (HMod.hMod b 64))
theorem
UInt16.toUInt8_shiftLeft
(a b : UInt16)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt8 (HShiftLeft.hShiftLeft a.toUInt8 b.toUInt8)
theorem
UInt32.toUInt8_shiftLeft
(a b : UInt32)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt8 (HShiftLeft.hShiftLeft a.toUInt8 b.toUInt8)
theorem
UInt32.toUInt16_shiftLeft
(a b : UInt32)
(hb : LT.lt b 16)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt16 (HShiftLeft.hShiftLeft a.toUInt16 b.toUInt16)
theorem
USize.toUInt8_shiftLeft
(a b : USize)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt8 (HShiftLeft.hShiftLeft a.toUInt8 b.toUInt8)
theorem
USize.toUInt16_shiftLeft
(a b : USize)
(hb : LT.lt b 16)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt16 (HShiftLeft.hShiftLeft a.toUInt16 b.toUInt16)
theorem
USize.toUInt32_shiftLeft
(a b : USize)
(hb : LT.lt b 32)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt32 (HShiftLeft.hShiftLeft a.toUInt32 b.toUInt32)
theorem
UInt64.toUInt8_shiftLeft
(a b : UInt64)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt8 (HShiftLeft.hShiftLeft a.toUInt8 b.toUInt8)
theorem
UInt64.toUInt16_shiftLeft
(a b : UInt64)
(hb : LT.lt b 16)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt16 (HShiftLeft.hShiftLeft a.toUInt16 b.toUInt16)
theorem
UInt64.toUInt32_shiftLeft
(a b : UInt64)
(hb : LT.lt b 32)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt32 (HShiftLeft.hShiftLeft a.toUInt32 b.toUInt32)
theorem
UInt64.toUSize_shiftLeft
(a b : UInt64)
(hb : LT.lt b.toNat System.Platform.numBits)
:
Eq (HShiftLeft.hShiftLeft a b).toUSize (HShiftLeft.hShiftLeft a.toUSize b.toUSize)
theorem
UInt16.toUInt8_shiftLeft_mod
(a b : UInt16)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 8)).toUInt8 (HShiftLeft.hShiftLeft a.toUInt8 b.toUInt8)
theorem
UInt32.toUInt8_shiftLeft_mod
(a b : UInt32)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 8)).toUInt8 (HShiftLeft.hShiftLeft a.toUInt8 b.toUInt8)
theorem
UInt32.toUInt16_shiftLeft_mod
(a b : UInt32)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 16)).toUInt16 (HShiftLeft.hShiftLeft a.toUInt16 b.toUInt16)
theorem
USize.toUInt8_shiftLeft_mod
(a b : USize)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 8)).toUInt8 (HShiftLeft.hShiftLeft a.toUInt8 b.toUInt8)
theorem
USize.toUInt16_shiftLeft_mod
(a b : USize)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 16)).toUInt16 (HShiftLeft.hShiftLeft a.toUInt16 b.toUInt16)
theorem
USize.toUInt32_shiftLeft_mod
(a b : USize)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 32)).toUInt32 (HShiftLeft.hShiftLeft a.toUInt32 b.toUInt32)
theorem
UInt64.toUInt8_shiftLeft_mod
(a b : UInt64)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 8)).toUInt8 (HShiftLeft.hShiftLeft a.toUInt8 b.toUInt8)
theorem
UInt64.toUInt16_shiftLeft_mod
(a b : UInt64)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 16)).toUInt16 (HShiftLeft.hShiftLeft a.toUInt16 b.toUInt16)
theorem
UInt64.toUInt32_shiftLeft_mod
(a b : UInt64)
:
Eq (HShiftLeft.hShiftLeft a (HMod.hMod b 32)).toUInt32 (HShiftLeft.hShiftLeft a.toUInt32 b.toUInt32)
theorem
UInt8.toUInt16_shiftLeft_of_lt
(a b : UInt8)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt16 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt16 b.toUInt16) 256)
theorem
UInt8.toUInt32_shiftLeft_of_lt
(a b : UInt8)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt32 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt32 b.toUInt32) 256)
theorem
UInt8.toUInt64_shiftLeft_of_lt
(a b : UInt8)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt64 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt64 b.toUInt64) 256)
theorem
UInt8.toUSize_shiftLeft_of_lt
(a b : UInt8)
(hb : LT.lt b 8)
:
Eq (HShiftLeft.hShiftLeft a b).toUSize (HMod.hMod (HShiftLeft.hShiftLeft a.toUSize b.toUSize) 256)
theorem
UInt16.toUInt32_shiftLeft_of_lt
(a b : UInt16)
(hb : LT.lt b 16)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt32 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt32 b.toUInt32) 65536)
theorem
UInt16.toUInt64_shiftLeft_of_lt
(a b : UInt16)
(hb : LT.lt b 16)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt64 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt64 b.toUInt64) 65536)
theorem
UInt16.toUSize_shiftLeft_of_lt
(a b : UInt16)
(hb : LT.lt b 16)
:
Eq (HShiftLeft.hShiftLeft a b).toUSize (HMod.hMod (HShiftLeft.hShiftLeft a.toUSize b.toUSize) 65536)
theorem
UInt32.toUInt64_shiftLeft_of_lt
(a b : UInt32)
(hb : LT.lt b 32)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt64 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt64 b.toUInt64) 4294967296)
theorem
UInt32.toUSize_shiftLeft_of_lt
(a b : UInt32)
(hb : LT.lt b 32)
:
Eq (HShiftLeft.hShiftLeft a b).toUSize (HMod.hMod (HShiftLeft.hShiftLeft a.toUSize b.toUSize) 4294967296)
theorem
USize.toUInt64_shiftLeft_of_lt
(a b : USize)
(hb : LT.lt b.toNat System.Platform.numBits)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt64 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt64 b.toUInt64) (UInt64.ofNat size))
theorem
UInt8.toUInt16_shiftLeft
(a b : UInt8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt16 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt16 (HMod.hMod b 8).toUInt16) 256)
theorem
UInt8.toUInt32_shiftLeft
(a b : UInt8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt32 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt32 (HMod.hMod b 8).toUInt32) 256)
theorem
UInt8.toUInt64_shiftLeft
(a b : UInt8)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt64 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt64 (HMod.hMod b 8).toUInt64) 256)
theorem
UInt8.toUSize_shiftLeft
(a b : UInt8)
:
Eq (HShiftLeft.hShiftLeft a b).toUSize (HMod.hMod (HShiftLeft.hShiftLeft a.toUSize (HMod.hMod b 8).toUSize) 256)
theorem
UInt16.toUInt32_shiftLeft
(a b : UInt16)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt32 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt32 (HMod.hMod b 16).toUInt32) 65536)
theorem
UInt16.toUInt64_shiftLeft
(a b : UInt16)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt64 (HMod.hMod (HShiftLeft.hShiftLeft a.toUInt64 (HMod.hMod b 16).toUInt64) 65536)
theorem
UInt16.toUSize_shiftLeft
(a b : UInt16)
:
Eq (HShiftLeft.hShiftLeft a b).toUSize (HMod.hMod (HShiftLeft.hShiftLeft a.toUSize (HMod.hMod b 16).toUSize) 65536)
theorem
UInt32.toUInt64_shiftLeft
(a b : UInt32)
:
Eq (HShiftLeft.hShiftLeft a b).toUInt64
(HMod.hMod (HShiftLeft.hShiftLeft a.toUInt64 (HMod.hMod b 32).toUInt64) 4294967296)
theorem
UInt32.toUSize_shiftLeft
(a b : UInt32)
:
Eq (HShiftLeft.hShiftLeft a b).toUSize (HMod.hMod (HShiftLeft.hShiftLeft a.toUSize (HMod.hMod b 32).toUSize) 4294967296)
theorem
UInt8.toFin_shiftRight
(a b : UInt8)
(hb : LT.lt b 8)
:
Eq (HShiftRight.hShiftRight a b).toFin (HShiftRight.hShiftRight a.toFin b.toFin)
theorem
UInt16.toFin_shiftRight
(a b : UInt16)
(hb : LT.lt b 16)
:
Eq (HShiftRight.hShiftRight a b).toFin (HShiftRight.hShiftRight a.toFin b.toFin)
theorem
UInt32.toFin_shiftRight
(a b : UInt32)
(hb : LT.lt b 32)
:
Eq (HShiftRight.hShiftRight a b).toFin (HShiftRight.hShiftRight a.toFin b.toFin)
theorem
UInt64.toFin_shiftRight
(a b : UInt64)
(hb : LT.lt b 64)
:
Eq (HShiftRight.hShiftRight a b).toFin (HShiftRight.hShiftRight a.toFin b.toFin)
theorem
USize.toFin_shiftRight
(a b : USize)
(hb : LT.lt b.toNat System.Platform.numBits)
:
Eq (HShiftRight.hShiftRight a b).toFin (HShiftRight.hShiftRight a.toFin b.toFin)
theorem
UInt8.toUInt16_shiftRight
(a b : UInt8)
:
Eq (HShiftRight.hShiftRight a b).toUInt16 (HShiftRight.hShiftRight a.toUInt16 (HMod.hMod b.toUInt16 8))
theorem
UInt8.toUInt32_shiftRight
(a b : UInt8)
:
Eq (HShiftRight.hShiftRight a b).toUInt32 (HShiftRight.hShiftRight a.toUInt32 (HMod.hMod b.toUInt32 8))
theorem
UInt8.toUInt64_shiftRight
(a b : UInt8)
:
Eq (HShiftRight.hShiftRight a b).toUInt64 (HShiftRight.hShiftRight a.toUInt64 (HMod.hMod b.toUInt64 8))
theorem
UInt8.toUSize_shiftRight
(a b : UInt8)
:
Eq (HShiftRight.hShiftRight a b).toUSize (HShiftRight.hShiftRight a.toUSize (HMod.hMod b.toUSize 8))
theorem
UInt16.toUInt32_shiftRight
(a b : UInt16)
:
Eq (HShiftRight.hShiftRight a b).toUInt32 (HShiftRight.hShiftRight a.toUInt32 (HMod.hMod b.toUInt32 16))
theorem
UInt16.toUInt64_shiftRight
(a b : UInt16)
:
Eq (HShiftRight.hShiftRight a b).toUInt64 (HShiftRight.hShiftRight a.toUInt64 (HMod.hMod b.toUInt64 16))
theorem
UInt16.toUSize_shiftRight
(a b : UInt16)
:
Eq (HShiftRight.hShiftRight a b).toUSize (HShiftRight.hShiftRight a.toUSize (HMod.hMod b.toUSize 16))
theorem
UInt32.toUInt64_shiftRight
(a b : UInt32)
:
Eq (HShiftRight.hShiftRight a b).toUInt64 (HShiftRight.hShiftRight a.toUInt64 (HMod.hMod b.toUInt64 32))
theorem
UInt32.toUSize_shiftRight
(a b : UInt32)
:
Eq (HShiftRight.hShiftRight a b).toUSize (HShiftRight.hShiftRight a.toUSize (HMod.hMod b.toUSize 32))
There is no reasonable statement forUInt16.toUInt8_shiftRight
; in fact for a b : UInt16
the
expression (a >>> b).toUInt8
is not a function of a.toUInt8
and b.toUInt8
.
theorem
UInt8.ofBitVec_not
(a : BitVec 8)
:
Eq { toBitVec := Complement.complement a } (Complement.complement { toBitVec := a })
theorem
UInt16.ofBitVec_not
(a : BitVec 16)
:
Eq { toBitVec := Complement.complement a } (Complement.complement { toBitVec := a })
theorem
UInt32.ofBitVec_not
(a : BitVec 32)
:
Eq { toBitVec := Complement.complement a } (Complement.complement { toBitVec := a })
theorem
UInt64.ofBitVec_not
(a : BitVec 64)
:
Eq { toBitVec := Complement.complement a } (Complement.complement { toBitVec := a })
theorem
USize.ofBitVec_not
(a : BitVec System.Platform.numBits)
:
Eq { toBitVec := Complement.complement a } (Complement.complement { toBitVec := a })
theorem
UInt8.ofBitVec_shiftLeft
(a : BitVec 8)
(b : Nat)
(hb : LT.lt b 8)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a b } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
UInt16.ofBitVec_shiftLeft
(a : BitVec 16)
(b : Nat)
(hb : LT.lt b 16)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a b } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
UInt32.ofBitVec_shiftLeft
(a : BitVec 32)
(b : Nat)
(hb : LT.lt b 32)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a b } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
UInt64.ofBitVec_shiftLeft
(a : BitVec 64)
(b : Nat)
(hb : LT.lt b 64)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a b } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
USize.ofBitVec_shiftLeft
(a : BitVec System.Platform.numBits)
(b : Nat)
(hb : LT.lt b System.Platform.numBits)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a b } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
UInt8.ofBitVec_shiftLeft_mod
(a : BitVec 8)
(b : Nat)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a (HMod.hMod b 8) } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
UInt16.ofBitVec_shiftLeft_mod
(a : BitVec 16)
(b : Nat)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a (HMod.hMod b 16) } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
UInt32.ofBitVec_shiftLeft_mod
(a : BitVec 32)
(b : Nat)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a (HMod.hMod b 32) } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
UInt64.ofBitVec_shiftLeft_mod
(a : BitVec 64)
(b : Nat)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a (HMod.hMod b 64) } (HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
USize.ofBitVec_shiftLeft_mod
(a : BitVec System.Platform.numBits)
(b : Nat)
:
Eq { toBitVec := HShiftLeft.hShiftLeft a (HMod.hMod b System.Platform.numBits) }
(HShiftLeft.hShiftLeft { toBitVec := a } (ofNat b))
theorem
UInt8.ofFin_shiftLeft
(a b : Fin size)
(hb : LT.lt b 8)
:
Eq (ofFin (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
UInt16.ofFin_shiftLeft
(a b : Fin size)
(hb : LT.lt b 16)
:
Eq (ofFin (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
UInt32.ofFin_shiftLeft
(a b : Fin size)
(hb : LT.lt b 32)
:
Eq (ofFin (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
UInt64.ofFin_shiftLeft
(a b : Fin size)
(hb : LT.lt b 64)
:
Eq (ofFin (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
USize.ofFin_shiftLeft
(a b : Fin size)
(hb : LT.lt b.val System.Platform.numBits)
:
Eq (ofFin (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
UInt8.ofFin_shiftLeft_mod
(a b : Fin size)
:
Eq (ofFin (HShiftLeft.hShiftLeft a (HMod.hMod b 8))) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
UInt16.ofFin_shiftLeft_mod
(a b : Fin size)
:
Eq (ofFin (HShiftLeft.hShiftLeft a (HMod.hMod b 16))) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
UInt32.ofFin_shiftLeft_mod
(a b : Fin size)
:
Eq (ofFin (HShiftLeft.hShiftLeft a (HMod.hMod b 32))) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
UInt64.ofFin_shiftLeft_mod
(a b : Fin size)
:
Eq (ofFin (HShiftLeft.hShiftLeft a (HMod.hMod b 64))) (HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
USize.ofFin_shiftLeft_mod
(a b : Fin size)
:
Eq (ofFin (HShiftLeft.hShiftLeft a (HMod.hMod b ⟨System.Platform.numBits, ⋯⟩)))
(HShiftLeft.hShiftLeft (ofFin a) (ofFin b))
theorem
UInt8.ofNat_shiftLeft
(a b : Nat)
(hb : LT.lt b 8)
:
Eq (ofNat (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofNat a) (ofNat b))
theorem
UInt16.ofNat_shiftLeft
(a b : Nat)
(hb : LT.lt b 16)
:
Eq (ofNat (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofNat a) (ofNat b))
theorem
UInt32.ofNat_shiftLeft
(a b : Nat)
(hb : LT.lt b 32)
:
Eq (ofNat (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofNat a) (ofNat b))
theorem
UInt64.ofNat_shiftLeft
(a b : Nat)
(hb : LT.lt b 64)
:
Eq (ofNat (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofNat a) (ofNat b))
theorem
USize.ofNat_shiftLeft
(a b : Nat)
(hb : LT.lt b System.Platform.numBits)
:
Eq (ofNat (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (ofNat a) (ofNat b))
theorem
UInt8.ofNatLT_shiftLeft
{a b : Nat}
(ha : LT.lt (HShiftLeft.hShiftLeft a b) size)
(hb : LT.lt b 8)
:
Eq (ofNatLT (HShiftLeft.hShiftLeft a b) ha) (HShiftLeft.hShiftLeft (ofNatLT a ⋯) (ofNatLT b ⋯))
theorem
UInt16.ofNatLT_shiftLeft
{a b : Nat}
(ha : LT.lt (HShiftLeft.hShiftLeft a b) size)
(hb : LT.lt b 16)
:
Eq (ofNatLT (HShiftLeft.hShiftLeft a b) ha) (HShiftLeft.hShiftLeft (ofNatLT a ⋯) (ofNatLT b ⋯))
theorem
UInt32.ofNatLT_shiftLeft
{a b : Nat}
(ha : LT.lt (HShiftLeft.hShiftLeft a b) size)
(hb : LT.lt b 32)
:
Eq (ofNatLT (HShiftLeft.hShiftLeft a b) ha) (HShiftLeft.hShiftLeft (ofNatLT a ⋯) (ofNatLT b ⋯))
theorem
UInt64.ofNatLT_shiftLeft
{a b : Nat}
(ha : LT.lt (HShiftLeft.hShiftLeft a b) size)
(hb : LT.lt b 64)
:
Eq (ofNatLT (HShiftLeft.hShiftLeft a b) ha) (HShiftLeft.hShiftLeft (ofNatLT a ⋯) (ofNatLT b ⋯))
theorem
USize.ofNatLT_shiftLeft
{a b : Nat}
(ha : LT.lt (HShiftLeft.hShiftLeft a b) size)
(hb : LT.lt b System.Platform.numBits)
:
Eq (ofNatLT (HShiftLeft.hShiftLeft a b) ha) (HShiftLeft.hShiftLeft (ofNatLT a ⋯) (ofNatLT b ⋯))
theorem
UInt8.ofBitVec_shiftRight
(a : BitVec 8)
(b : Nat)
(hb : LT.lt b 8)
:
Eq { toBitVec := HShiftRight.hShiftRight a b } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
UInt16.ofBitVec_shiftRight
(a : BitVec 16)
(b : Nat)
(hb : LT.lt b 16)
:
Eq { toBitVec := HShiftRight.hShiftRight a b } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
UInt32.ofBitVec_shiftRight
(a : BitVec 32)
(b : Nat)
(hb : LT.lt b 32)
:
Eq { toBitVec := HShiftRight.hShiftRight a b } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
UInt64.ofBitVec_shiftRight
(a : BitVec 64)
(b : Nat)
(hb : LT.lt b 64)
:
Eq { toBitVec := HShiftRight.hShiftRight a b } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
USize.ofBitVec_shiftRight
(a : BitVec System.Platform.numBits)
(b : Nat)
(hb : LT.lt b System.Platform.numBits)
:
Eq { toBitVec := HShiftRight.hShiftRight a b } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
UInt8.ofBitVec_shiftRight_mod
(a : BitVec 8)
(b : Nat)
:
Eq { toBitVec := HShiftRight.hShiftRight a (HMod.hMod b 8) } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
UInt16.ofBitVec_shiftRight_mod
(a : BitVec 16)
(b : Nat)
:
Eq { toBitVec := HShiftRight.hShiftRight a (HMod.hMod b 16) } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
UInt32.ofBitVec_shiftRight_mod
(a : BitVec 32)
(b : Nat)
:
Eq { toBitVec := HShiftRight.hShiftRight a (HMod.hMod b 32) } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
UInt64.ofBitVec_shiftRight_mod
(a : BitVec 64)
(b : Nat)
:
Eq { toBitVec := HShiftRight.hShiftRight a (HMod.hMod b 64) } (HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
USize.ofBitVec_shiftRight_mod
(a : BitVec System.Platform.numBits)
(b : Nat)
:
Eq { toBitVec := HShiftRight.hShiftRight a (HMod.hMod b System.Platform.numBits) }
(HShiftRight.hShiftRight { toBitVec := a } (ofNat b))
theorem
UInt8.ofFin_shiftRight
(a b : Fin size)
(hb : LT.lt b 8)
:
Eq (ofFin (HShiftRight.hShiftRight a b)) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
UInt16.ofFin_shiftRight
(a b : Fin size)
(hb : LT.lt b 16)
:
Eq (ofFin (HShiftRight.hShiftRight a b)) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
UInt32.ofFin_shiftRight
(a b : Fin size)
(hb : LT.lt b 32)
:
Eq (ofFin (HShiftRight.hShiftRight a b)) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
UInt64.ofFin_shiftRight
(a b : Fin size)
(hb : LT.lt b 64)
:
Eq (ofFin (HShiftRight.hShiftRight a b)) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
USize.ofFin_shiftRight
(a b : Fin size)
(hb : LT.lt b.val System.Platform.numBits)
:
Eq (ofFin (HShiftRight.hShiftRight a b)) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
UInt8.ofFin_shiftRight_mod
(a b : Fin size)
:
Eq (ofFin (HShiftRight.hShiftRight a (HMod.hMod b 8))) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
UInt16.ofFin_shiftRight_mod
(a b : Fin size)
:
Eq (ofFin (HShiftRight.hShiftRight a (HMod.hMod b 16))) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
UInt32.ofFin_shiftRight_mod
(a b : Fin size)
:
Eq (ofFin (HShiftRight.hShiftRight a (HMod.hMod b 32))) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
UInt64.ofFin_shiftRight_mod
(a b : Fin size)
:
Eq (ofFin (HShiftRight.hShiftRight a (HMod.hMod b 64))) (HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
USize.ofFin_shiftRight_mod
(a b : Fin size)
:
Eq (ofFin (HShiftRight.hShiftRight a (HMod.hMod b ⟨System.Platform.numBits, ⋯⟩)))
(HShiftRight.hShiftRight (ofFin a) (ofFin b))
theorem
instLawfulCommIdentityUInt8HOrOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt8) => HOr.hOr x1 x2) 0
theorem
instLawfulCommIdentityUInt16HOrOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt16) => HOr.hOr x1 x2) 0
theorem
instLawfulCommIdentityUInt32HOrOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt32) => HOr.hOr x1 x2) 0
theorem
instLawfulCommIdentityUInt64HOrOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt64) => HOr.hOr x1 x2) 0
theorem
instLawfulCommIdentityUSizeHOrOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : USize) => HOr.hOr x1 x2) 0
theorem
instLawfulCommIdentityUInt8HAndNegOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt8) => HAnd.hAnd x1 x2) (-1)
theorem
instLawfulCommIdentityUInt16HAndNegOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt16) => HAnd.hAnd x1 x2) (-1)
theorem
instLawfulCommIdentityUInt32HAndNegOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt32) => HAnd.hAnd x1 x2) (-1)
theorem
instLawfulCommIdentityUInt64HAndNegOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt64) => HAnd.hAnd x1 x2) (-1)
theorem
instLawfulCommIdentityUSizeHAndNegOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : USize) => HAnd.hAnd x1 x2) (-1)
theorem
instLawfulCommIdentityUInt8HXorOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt8) => HXor.hXor x1 x2) 0
theorem
instLawfulCommIdentityUInt16HXorOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt16) => HXor.hXor x1 x2) 0
theorem
instLawfulCommIdentityUInt32HXorOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt32) => HXor.hXor x1 x2) 0
theorem
instLawfulCommIdentityUInt64HXorOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : UInt64) => HXor.hXor x1 x2) 0
theorem
instLawfulCommIdentityUSizeHXorOfNat :
Std.LawfulCommIdentity (fun (x1 x2 : USize) => HXor.hXor x1 x2) 0
theorem
UInt8.not_inj
{a b : UInt8}
:
Iff (Eq (Complement.complement a) (Complement.complement b)) (Eq a b)
theorem
UInt16.not_inj
{a b : UInt16}
:
Iff (Eq (Complement.complement a) (Complement.complement b)) (Eq a b)
theorem
UInt32.not_inj
{a b : UInt32}
:
Iff (Eq (Complement.complement a) (Complement.complement b)) (Eq a b)
theorem
UInt64.not_inj
{a b : UInt64}
:
Iff (Eq (Complement.complement a) (Complement.complement b)) (Eq a b)
theorem
USize.not_inj
{a b : USize}
:
Iff (Eq (Complement.complement a) (Complement.complement b)) (Eq a b)
theorem
UInt8.not_eq_comm
{a b : UInt8}
:
Iff (Eq (Complement.complement a) b) (Eq a (Complement.complement b))
theorem
UInt16.not_eq_comm
{a b : UInt16}
:
Iff (Eq (Complement.complement a) b) (Eq a (Complement.complement b))
theorem
UInt32.not_eq_comm
{a b : UInt32}
:
Iff (Eq (Complement.complement a) b) (Eq a (Complement.complement b))
theorem
UInt64.not_eq_comm
{a b : UInt64}
:
Iff (Eq (Complement.complement a) b) (Eq a (Complement.complement b))
theorem
USize.not_eq_comm
{a b : USize}
:
Iff (Eq (Complement.complement a) b) (Eq a (Complement.complement b))
theorem
UInt8.not_xor
{a b : UInt8}
:
Eq (HXor.hXor (Complement.complement a) b) (Complement.complement (HXor.hXor a b))
theorem
UInt16.not_xor
{a b : UInt16}
:
Eq (HXor.hXor (Complement.complement a) b) (Complement.complement (HXor.hXor a b))
theorem
UInt32.not_xor
{a b : UInt32}
:
Eq (HXor.hXor (Complement.complement a) b) (Complement.complement (HXor.hXor a b))
theorem
UInt64.not_xor
{a b : UInt64}
:
Eq (HXor.hXor (Complement.complement a) b) (Complement.complement (HXor.hXor a b))
theorem
USize.not_xor
{a b : USize}
:
Eq (HXor.hXor (Complement.complement a) b) (Complement.complement (HXor.hXor a b))
theorem
UInt8.xor_not
{a b : UInt8}
:
Eq (HXor.hXor a (Complement.complement b)) (Complement.complement (HXor.hXor a b))
theorem
UInt16.xor_not
{a b : UInt16}
:
Eq (HXor.hXor a (Complement.complement b)) (Complement.complement (HXor.hXor a b))
theorem
UInt32.xor_not
{a b : UInt32}
:
Eq (HXor.hXor a (Complement.complement b)) (Complement.complement (HXor.hXor a b))
theorem
UInt64.xor_not
{a b : UInt64}
:
Eq (HXor.hXor a (Complement.complement b)) (Complement.complement (HXor.hXor a b))
theorem
USize.xor_not
{a b : USize}
:
Eq (HXor.hXor a (Complement.complement b)) (Complement.complement (HXor.hXor a b))
theorem
UInt8.shiftLeft_xor
{a b c : UInt8}
:
Eq (HShiftLeft.hShiftLeft (HXor.hXor a b) c) (HXor.hXor (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt16.shiftLeft_xor
{a b c : UInt16}
:
Eq (HShiftLeft.hShiftLeft (HXor.hXor a b) c) (HXor.hXor (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt32.shiftLeft_xor
{a b c : UInt32}
:
Eq (HShiftLeft.hShiftLeft (HXor.hXor a b) c) (HXor.hXor (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt64.shiftLeft_xor
{a b c : UInt64}
:
Eq (HShiftLeft.hShiftLeft (HXor.hXor a b) c) (HXor.hXor (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
USize.shiftLeft_xor
{a b c : USize}
:
Eq (HShiftLeft.hShiftLeft (HXor.hXor a b) c) (HXor.hXor (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt8.shiftLeft_and
{a b c : UInt8}
:
Eq (HShiftLeft.hShiftLeft (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt16.shiftLeft_and
{a b c : UInt16}
:
Eq (HShiftLeft.hShiftLeft (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt32.shiftLeft_and
{a b c : UInt32}
:
Eq (HShiftLeft.hShiftLeft (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt64.shiftLeft_and
{a b c : UInt64}
:
Eq (HShiftLeft.hShiftLeft (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
USize.shiftLeft_and
{a b c : USize}
:
Eq (HShiftLeft.hShiftLeft (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt8.shiftLeft_or
{a b c : UInt8}
:
Eq (HShiftLeft.hShiftLeft (HOr.hOr a b) c) (HOr.hOr (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt16.shiftLeft_or
{a b c : UInt16}
:
Eq (HShiftLeft.hShiftLeft (HOr.hOr a b) c) (HOr.hOr (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt32.shiftLeft_or
{a b c : UInt32}
:
Eq (HShiftLeft.hShiftLeft (HOr.hOr a b) c) (HOr.hOr (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt64.shiftLeft_or
{a b c : UInt64}
:
Eq (HShiftLeft.hShiftLeft (HOr.hOr a b) c) (HOr.hOr (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
USize.shiftLeft_or
{a b c : USize}
:
Eq (HShiftLeft.hShiftLeft (HOr.hOr a b) c) (HOr.hOr (HShiftLeft.hShiftLeft a c) (HShiftLeft.hShiftLeft b c))
theorem
UInt8.shiftLeft_add_of_toNat_lt
{a b c : UInt8}
(h : LT.lt (HAdd.hAdd b.toNat c.toNat) 8)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
UInt16.shiftLeft_add_of_toNat_lt
{a b c : UInt16}
(h : LT.lt (HAdd.hAdd b.toNat c.toNat) 16)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
UInt32.shiftLeft_add_of_toNat_lt
{a b c : UInt32}
(h : LT.lt (HAdd.hAdd b.toNat c.toNat) 32)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
UInt64.shiftLeft_add_of_toNat_lt
{a b c : UInt64}
(h : LT.lt (HAdd.hAdd b.toNat c.toNat) 64)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
USize.shiftLeft_add_of_toNat_lt
{a b c : USize}
(h : LT.lt (HAdd.hAdd b.toNat c.toNat) System.Platform.numBits)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
UInt8.shiftLeft_add
{a b c : UInt8}
(hb : LT.lt b 8)
(hc : LT.lt c 8)
(hbc : LT.lt (HAdd.hAdd b c) 8)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
UInt16.shiftLeft_add
{a b c : UInt16}
(hb : LT.lt b 16)
(hc : LT.lt c 16)
(hbc : LT.lt (HAdd.hAdd b c) 16)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
UInt32.shiftLeft_add
{a b c : UInt32}
(hb : LT.lt b 32)
(hc : LT.lt c 32)
(hbc : LT.lt (HAdd.hAdd b c) 32)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
UInt64.shiftLeft_add
{a b c : UInt64}
(hb : LT.lt b 64)
(hc : LT.lt c 64)
(hbc : LT.lt (HAdd.hAdd b c) 64)
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
USize.shiftLeft_add
{a b c : USize}
(hb : LT.lt b (ofNat System.Platform.numBits))
(hc : LT.lt c (ofNat System.Platform.numBits))
(hbc : LT.lt (HAdd.hAdd b c) (ofNat System.Platform.numBits))
:
Eq (HShiftLeft.hShiftLeft a (HAdd.hAdd b c)) (HShiftLeft.hShiftLeft (HShiftLeft.hShiftLeft a b) c)
theorem
UInt8.neg_one_shiftLeft_and_shiftLeft
{a b : UInt8}
:
Eq (HAnd.hAnd (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft a b)
theorem
UInt16.neg_one_shiftLeft_and_shiftLeft
{a b : UInt16}
:
Eq (HAnd.hAnd (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft a b)
theorem
UInt32.neg_one_shiftLeft_and_shiftLeft
{a b : UInt32}
:
Eq (HAnd.hAnd (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft a b)
theorem
UInt64.neg_one_shiftLeft_and_shiftLeft
{a b : UInt64}
:
Eq (HAnd.hAnd (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft a b)
theorem
USize.neg_one_shiftLeft_and_shiftLeft
{a b : USize}
:
Eq (HAnd.hAnd (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft a b)
theorem
UInt8.neg_one_shiftLeft_or_shiftLeft
{a b : UInt8}
:
Eq (HOr.hOr (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (-1) b)
theorem
UInt16.neg_one_shiftLeft_or_shiftLeft
{a b : UInt16}
:
Eq (HOr.hOr (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (-1) b)
theorem
UInt32.neg_one_shiftLeft_or_shiftLeft
{a b : UInt32}
:
Eq (HOr.hOr (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (-1) b)
theorem
UInt64.neg_one_shiftLeft_or_shiftLeft
{a b : UInt8}
:
Eq (HOr.hOr (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (-1) b)
theorem
USize.neg_one_shiftLeft_or_shiftLeft
{a b : USize}
:
Eq (HOr.hOr (HShiftLeft.hShiftLeft (-1) b) (HShiftLeft.hShiftLeft a b)) (HShiftLeft.hShiftLeft (-1) b)
theorem
UInt8.shiftRight_xor
{a b c : UInt8}
:
Eq (HShiftRight.hShiftRight (HXor.hXor a b) c) (HXor.hXor (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt16.shiftRight_xor
{a b c : UInt16}
:
Eq (HShiftRight.hShiftRight (HXor.hXor a b) c) (HXor.hXor (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt32.shiftRight_xor
{a b c : UInt32}
:
Eq (HShiftRight.hShiftRight (HXor.hXor a b) c) (HXor.hXor (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt64.shiftRight_xor
{a b c : UInt64}
:
Eq (HShiftRight.hShiftRight (HXor.hXor a b) c) (HXor.hXor (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
USize.shiftRight_xor
{a b c : USize}
:
Eq (HShiftRight.hShiftRight (HXor.hXor a b) c) (HXor.hXor (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt8.shiftRight_and
{a b c : UInt8}
:
Eq (HShiftRight.hShiftRight (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt16.shiftRight_and
{a b c : UInt16}
:
Eq (HShiftRight.hShiftRight (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt32.shiftRight_and
{a b c : UInt32}
:
Eq (HShiftRight.hShiftRight (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt64.shiftRight_and
{a b c : UInt64}
:
Eq (HShiftRight.hShiftRight (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
USize.shiftRight_and
{a b c : USize}
:
Eq (HShiftRight.hShiftRight (HAnd.hAnd a b) c) (HAnd.hAnd (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt8.shiftRight_or
{a b c : UInt8}
:
Eq (HShiftRight.hShiftRight (HOr.hOr a b) c) (HOr.hOr (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt16.shiftRight_or
{a b c : UInt16}
:
Eq (HShiftRight.hShiftRight (HOr.hOr a b) c) (HOr.hOr (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt32.shiftRight_or
{a b c : UInt32}
:
Eq (HShiftRight.hShiftRight (HOr.hOr a b) c) (HOr.hOr (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
UInt64.shiftRight_or
{a b c : UInt64}
:
Eq (HShiftRight.hShiftRight (HOr.hOr a b) c) (HOr.hOr (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))
theorem
USize.shiftRight_or
{a b c : USize}
:
Eq (HShiftRight.hShiftRight (HOr.hOr a b) c) (HOr.hOr (HShiftRight.hShiftRight a c) (HShiftRight.hShiftRight b c))