Documentation

Init.Data.UInt.Bitwise

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[deprecated UInt8.toNat_and (since := "2024-11-28")]
    @[deprecated UInt16.toNat_and (since := "2024-11-28")]
    @[deprecated UInt32.toNat_and (since := "2024-11-28")]
    @[deprecated UInt64.toNat_and (since := "2024-11-28")]
    @[deprecated USize.toNat_and (since := "2024-11-28")]

    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.ofFin_and (a b : Fin size) :
    theorem UInt16.ofFin_and (a b : Fin size) :
    theorem UInt32.ofFin_and (a b : Fin size) :
    theorem UInt64.ofFin_and (a b : Fin size) :
    theorem USize.ofFin_and (a b : Fin size) :
    theorem UInt8.ofBitVec_and (a b : BitVec 8) :
    Eq { toBitVec := HAnd.hAnd a b } (HAnd.hAnd { toBitVec := a } { toBitVec := b })
    theorem UInt16.ofBitVec_and (a b : BitVec 16) :
    Eq { toBitVec := HAnd.hAnd a b } (HAnd.hAnd { toBitVec := a } { toBitVec := b })
    theorem UInt32.ofBitVec_and (a b : BitVec 32) :
    Eq { toBitVec := HAnd.hAnd a b } (HAnd.hAnd { toBitVec := a } { toBitVec := b })
    theorem UInt64.ofBitVec_and (a b : BitVec 64) :
    Eq { toBitVec := HAnd.hAnd a b } (HAnd.hAnd { toBitVec := a } { toBitVec := b })
    theorem USize.ofBitVec_and (a b : BitVec System.Platform.numBits) :
    Eq { toBitVec := HAnd.hAnd a b } (HAnd.hAnd { toBitVec := a } { toBitVec := b })
    theorem UInt8.ofNat_and (a b : Nat) :
    theorem UInt16.ofNat_and (a b : Nat) :
    theorem UInt32.ofNat_and (a b : Nat) :
    theorem UInt64.ofNat_and (a b : Nat) :
    theorem USize.ofNat_and (a b : Nat) :
    theorem UInt8.ofNatLT_and (a b : Nat) (ha : LT.lt a (HPow.hPow 2 8)) (hb : LT.lt b (HPow.hPow 2 8)) :
    Eq (ofNatLT (HAnd.hAnd a b) ⋯) (HAnd.hAnd (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt16.ofNatLT_and (a b : Nat) (ha : LT.lt a (HPow.hPow 2 16)) (hb : LT.lt b (HPow.hPow 2 16)) :
    Eq (ofNatLT (HAnd.hAnd a b) ⋯) (HAnd.hAnd (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt32.ofNatLT_and (a b : Nat) (ha : LT.lt a (HPow.hPow 2 32)) (hb : LT.lt b (HPow.hPow 2 32)) :
    Eq (ofNatLT (HAnd.hAnd a b) ⋯) (HAnd.hAnd (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt64.ofNatLT_and (a b : Nat) (ha : LT.lt a (HPow.hPow 2 64)) (hb : LT.lt b (HPow.hPow 2 64)) :
    Eq (ofNatLT (HAnd.hAnd a b) ⋯) (HAnd.hAnd (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt8.ofFin_or (a b : Fin size) :
    Eq (ofFin (HOr.hOr a b)) (HOr.hOr (ofFin a) (ofFin b))
    theorem UInt16.ofFin_or (a b : Fin size) :
    Eq (ofFin (HOr.hOr a b)) (HOr.hOr (ofFin a) (ofFin b))
    theorem UInt32.ofFin_or (a b : Fin size) :
    Eq (ofFin (HOr.hOr a b)) (HOr.hOr (ofFin a) (ofFin b))
    theorem UInt64.ofFin_or (a b : Fin size) :
    Eq (ofFin (HOr.hOr a b)) (HOr.hOr (ofFin a) (ofFin b))
    theorem USize.ofFin_or (a b : Fin size) :
    Eq (ofFin (HOr.hOr a b)) (HOr.hOr (ofFin a) (ofFin b))
    theorem UInt8.ofBitVec_or (a b : BitVec 8) :
    Eq { toBitVec := HOr.hOr a b } (HOr.hOr { toBitVec := a } { toBitVec := b })
    theorem UInt16.ofBitVec_or (a b : BitVec 16) :
    Eq { toBitVec := HOr.hOr a b } (HOr.hOr { toBitVec := a } { toBitVec := b })
    theorem UInt32.ofBitVec_or (a b : BitVec 32) :
    Eq { toBitVec := HOr.hOr a b } (HOr.hOr { toBitVec := a } { toBitVec := b })
    theorem UInt64.ofBitVec_or (a b : BitVec 64) :
    Eq { toBitVec := HOr.hOr a b } (HOr.hOr { toBitVec := a } { toBitVec := b })
    theorem USize.ofBitVec_or (a b : BitVec System.Platform.numBits) :
    Eq { toBitVec := HOr.hOr a b } (HOr.hOr { toBitVec := a } { toBitVec := b })
    theorem UInt8.ofNat_or (a b : Nat) :
    Eq (ofNat (HOr.hOr a b)) (HOr.hOr (ofNat a) (ofNat b))
    theorem UInt16.ofNat_or (a b : Nat) :
    Eq (ofNat (HOr.hOr a b)) (HOr.hOr (ofNat a) (ofNat b))
    theorem UInt32.ofNat_or (a b : Nat) :
    Eq (ofNat (HOr.hOr a b)) (HOr.hOr (ofNat a) (ofNat b))
    theorem UInt64.ofNat_or (a b : Nat) :
    Eq (ofNat (HOr.hOr a b)) (HOr.hOr (ofNat a) (ofNat b))
    theorem USize.ofNat_or (a b : Nat) :
    Eq (ofNat (HOr.hOr a b)) (HOr.hOr (ofNat a) (ofNat b))
    theorem UInt8.ofNatLT_or (a b : Nat) (ha : LT.lt a (HPow.hPow 2 8)) (hb : LT.lt b (HPow.hPow 2 8)) :
    Eq (ofNatLT (HOr.hOr a b) ⋯) (HOr.hOr (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt16.ofNatLT_or (a b : Nat) (ha : LT.lt a (HPow.hPow 2 16)) (hb : LT.lt b (HPow.hPow 2 16)) :
    Eq (ofNatLT (HOr.hOr a b) ⋯) (HOr.hOr (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt32.ofNatLT_or (a b : Nat) (ha : LT.lt a (HPow.hPow 2 32)) (hb : LT.lt b (HPow.hPow 2 32)) :
    Eq (ofNatLT (HOr.hOr a b) ⋯) (HOr.hOr (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt64.ofNatLT_or (a b : Nat) (ha : LT.lt a (HPow.hPow 2 64)) (hb : LT.lt b (HPow.hPow 2 64)) :
    Eq (ofNatLT (HOr.hOr a b) ⋯) (HOr.hOr (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt8.ofFin_xor (a b : Fin size) :
    theorem UInt16.ofFin_xor (a b : Fin size) :
    theorem UInt32.ofFin_xor (a b : Fin size) :
    theorem UInt64.ofFin_xor (a b : Fin size) :
    theorem USize.ofFin_xor (a b : Fin size) :
    theorem UInt8.ofBitVec_xor (a b : BitVec 8) :
    Eq { toBitVec := HXor.hXor a b } (HXor.hXor { toBitVec := a } { toBitVec := b })
    theorem UInt16.ofBitVec_xor (a b : BitVec 16) :
    Eq { toBitVec := HXor.hXor a b } (HXor.hXor { toBitVec := a } { toBitVec := b })
    theorem UInt32.ofBitVec_xor (a b : BitVec 32) :
    Eq { toBitVec := HXor.hXor a b } (HXor.hXor { toBitVec := a } { toBitVec := b })
    theorem UInt64.ofBitVec_xor (a b : BitVec 64) :
    Eq { toBitVec := HXor.hXor a b } (HXor.hXor { toBitVec := a } { toBitVec := b })
    theorem USize.ofBitVec_xor (a b : BitVec System.Platform.numBits) :
    Eq { toBitVec := HXor.hXor a b } (HXor.hXor { toBitVec := a } { toBitVec := b })
    theorem UInt8.ofNat_xor (a b : Nat) :
    theorem UInt16.ofNat_xor (a b : Nat) :
    theorem UInt32.ofNat_xor (a b : Nat) :
    theorem UInt64.ofNat_xor (a b : Nat) :
    theorem USize.ofNat_xor (a b : Nat) :
    theorem UInt8.ofNatLT_xor (a b : Nat) (ha : LT.lt a (HPow.hPow 2 8)) (hb : LT.lt b (HPow.hPow 2 8)) :
    Eq (ofNatLT (HXor.hXor a b) ⋯) (HXor.hXor (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt16.ofNatLT_xor (a b : Nat) (ha : LT.lt a (HPow.hPow 2 16)) (hb : LT.lt b (HPow.hPow 2 16)) :
    Eq (ofNatLT (HXor.hXor a b) ⋯) (HXor.hXor (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt32.ofNatLT_xor (a b : Nat) (ha : LT.lt a (HPow.hPow 2 32)) (hb : LT.lt b (HPow.hPow 2 32)) :
    Eq (ofNatLT (HXor.hXor a b) ⋯) (HXor.hXor (ofNatLT a ha) (ofNatLT b hb))
    theorem UInt64.ofNatLT_xor (a b : Nat) (ha : LT.lt a (HPow.hPow 2 64)) (hb : LT.lt b (HPow.hPow 2 64)) :
    Eq (ofNatLT (HXor.hXor a b) ⋯) (HXor.hXor (ofNatLT a ha) (ofNatLT b hb))
    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 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 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 UInt8.ofNatLT_shiftLeft {a b : Nat} (ha : LT.lt (HShiftLeft.hShiftLeft a b) size) (hb : LT.lt b 8) :
    theorem UInt16.ofNatLT_shiftLeft {a b : Nat} (ha : LT.lt (HShiftLeft.hShiftLeft a b) size) (hb : LT.lt b 16) :
    theorem UInt32.ofNatLT_shiftLeft {a b : Nat} (ha : LT.lt (HShiftLeft.hShiftLeft a b) size) (hb : LT.lt b 32) :
    theorem UInt64.ofNatLT_shiftLeft {a b : Nat} (ha : LT.lt (HShiftLeft.hShiftLeft a b) size) (hb : LT.lt b 64) :
    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 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 UInt8.or_assoc (a b c : UInt8) :
    Eq (HOr.hOr (HOr.hOr a b) c) (HOr.hOr a (HOr.hOr b c))
    theorem UInt16.or_assoc (a b c : UInt16) :
    Eq (HOr.hOr (HOr.hOr a b) c) (HOr.hOr a (HOr.hOr b c))
    theorem UInt32.or_assoc (a b c : UInt32) :
    Eq (HOr.hOr (HOr.hOr a b) c) (HOr.hOr a (HOr.hOr b c))
    theorem UInt64.or_assoc (a b c : UInt64) :
    Eq (HOr.hOr (HOr.hOr a b) c) (HOr.hOr a (HOr.hOr b c))
    theorem USize.or_assoc (a b c : USize) :
    Eq (HOr.hOr (HOr.hOr a b) c) (HOr.hOr a (HOr.hOr b c))
    theorem UInt8.or_comm (a b : UInt8) :
    Eq (HOr.hOr a b) (HOr.hOr b a)
    theorem UInt16.or_comm (a b : UInt16) :
    Eq (HOr.hOr a b) (HOr.hOr b a)
    theorem UInt32.or_comm (a b : UInt32) :
    Eq (HOr.hOr a b) (HOr.hOr b a)
    theorem UInt64.or_comm (a b : UInt64) :
    Eq (HOr.hOr a b) (HOr.hOr b a)
    theorem USize.or_comm (a b : USize) :
    Eq (HOr.hOr a b) (HOr.hOr b a)
    theorem UInt8.or_self {a : UInt8} :
    Eq (HOr.hOr a a) a
    theorem UInt16.or_self {a : UInt16} :
    Eq (HOr.hOr a a) a
    theorem UInt32.or_self {a : UInt32} :
    Eq (HOr.hOr a a) a
    theorem UInt64.or_self {a : UInt64} :
    Eq (HOr.hOr a a) a
    theorem USize.or_self {a : USize} :
    Eq (HOr.hOr a a) a
    theorem UInt8.or_zero {a : UInt8} :
    Eq (HOr.hOr a 0) a
    theorem UInt16.or_zero {a : UInt16} :
    Eq (HOr.hOr a 0) a
    theorem UInt32.or_zero {a : UInt32} :
    Eq (HOr.hOr a 0) a
    theorem UInt64.or_zero {a : UInt64} :
    Eq (HOr.hOr a 0) a
    theorem USize.or_zero {a : USize} :
    Eq (HOr.hOr a 0) a
    theorem UInt8.zero_or {a : UInt8} :
    Eq (HOr.hOr 0 a) a
    theorem UInt16.zero_or {a : UInt16} :
    Eq (HOr.hOr 0 a) a
    theorem UInt32.zero_or {a : UInt32} :
    Eq (HOr.hOr 0 a) a
    theorem UInt64.zero_or {a : UInt64} :
    Eq (HOr.hOr 0 a) a
    theorem USize.zero_or {a : USize} :
    Eq (HOr.hOr 0 a) a
    theorem UInt8.neg_one_or {a : UInt8} :
    Eq (HOr.hOr (-1) a) (-1)
    theorem UInt16.neg_one_or {a : UInt16} :
    Eq (HOr.hOr (-1) a) (-1)
    theorem UInt32.neg_one_or {a : UInt32} :
    Eq (HOr.hOr (-1) a) (-1)
    theorem UInt64.neg_one_or {a : UInt64} :
    Eq (HOr.hOr (-1) a) (-1)
    theorem USize.neg_one_or {a : USize} :
    Eq (HOr.hOr (-1) a) (-1)
    theorem UInt8.or_neg_one {a : UInt8} :
    Eq (HOr.hOr a (-1)) (-1)
    theorem UInt16.or_neg_one {a : UInt16} :
    Eq (HOr.hOr a (-1)) (-1)
    theorem UInt32.or_neg_one {a : UInt32} :
    Eq (HOr.hOr a (-1)) (-1)
    theorem UInt64.or_neg_one {a : UInt64} :
    Eq (HOr.hOr a (-1)) (-1)
    theorem USize.or_neg_one {a : USize} :
    Eq (HOr.hOr a (-1)) (-1)
    theorem UInt8.or_eq_zero_iff {a b : UInt8} :
    Iff (Eq (HOr.hOr a b) 0) (And (Eq a 0) (Eq b 0))
    theorem UInt16.or_eq_zero_iff {a b : UInt16} :
    Iff (Eq (HOr.hOr a b) 0) (And (Eq a 0) (Eq b 0))
    theorem UInt32.or_eq_zero_iff {a b : UInt32} :
    Iff (Eq (HOr.hOr a b) 0) (And (Eq a 0) (Eq b 0))
    theorem UInt64.or_eq_zero_iff {a b : UInt64} :
    Iff (Eq (HOr.hOr a b) 0) (And (Eq a 0) (Eq b 0))
    theorem USize.or_eq_zero_iff {a b : USize} :
    Iff (Eq (HOr.hOr a b) 0) (And (Eq a 0) (Eq b 0))
    theorem UInt8.and_assoc (a b c : UInt8) :
    theorem UInt16.and_assoc (a b c : UInt16) :
    theorem UInt32.and_assoc (a b c : UInt32) :
    theorem UInt64.and_assoc (a b c : UInt64) :
    theorem USize.and_assoc (a b c : USize) :
    theorem UInt8.and_comm (a b : UInt8) :
    Eq (HAnd.hAnd a b) (HAnd.hAnd b a)
    theorem UInt16.and_comm (a b : UInt16) :
    Eq (HAnd.hAnd a b) (HAnd.hAnd b a)
    theorem UInt32.and_comm (a b : UInt32) :
    Eq (HAnd.hAnd a b) (HAnd.hAnd b a)
    theorem UInt64.and_comm (a b : UInt64) :
    Eq (HAnd.hAnd a b) (HAnd.hAnd b a)
    theorem USize.and_comm (a b : USize) :
    Eq (HAnd.hAnd a b) (HAnd.hAnd b a)
    theorem UInt8.and_self {a : UInt8} :
    Eq (HAnd.hAnd a a) a
    theorem UInt16.and_self {a : UInt16} :
    Eq (HAnd.hAnd a a) a
    theorem UInt32.and_self {a : UInt32} :
    Eq (HAnd.hAnd a a) a
    theorem UInt64.and_self {a : UInt64} :
    Eq (HAnd.hAnd a a) a
    theorem USize.and_self {a : USize} :
    Eq (HAnd.hAnd a a) a
    theorem UInt8.and_zero {a : UInt8} :
    Eq (HAnd.hAnd a 0) 0
    theorem UInt16.and_zero {a : UInt16} :
    Eq (HAnd.hAnd a 0) 0
    theorem UInt32.and_zero {a : UInt32} :
    Eq (HAnd.hAnd a 0) 0
    theorem UInt64.and_zero {a : UInt64} :
    Eq (HAnd.hAnd a 0) 0
    theorem USize.and_zero {a : USize} :
    Eq (HAnd.hAnd a 0) 0
    theorem UInt8.zero_and {a : UInt8} :
    Eq (HAnd.hAnd 0 a) 0
    theorem UInt16.zero_and {a : UInt16} :
    Eq (HAnd.hAnd 0 a) 0
    theorem UInt32.zero_and {a : UInt32} :
    Eq (HAnd.hAnd 0 a) 0
    theorem UInt64.zero_and {a : UInt64} :
    Eq (HAnd.hAnd 0 a) 0
    theorem USize.zero_and {a : USize} :
    Eq (HAnd.hAnd 0 a) 0
    theorem UInt8.neg_one_and {a : UInt8} :
    Eq (HAnd.hAnd (-1) a) a
    theorem UInt16.neg_one_and {a : UInt16} :
    Eq (HAnd.hAnd (-1) a) a
    theorem UInt32.neg_one_and {a : UInt32} :
    Eq (HAnd.hAnd (-1) a) a
    theorem UInt64.neg_one_and {a : UInt64} :
    Eq (HAnd.hAnd (-1) a) a
    theorem USize.neg_one_and {a : USize} :
    Eq (HAnd.hAnd (-1) a) a
    theorem UInt8.and_neg_one {a : UInt8} :
    Eq (HAnd.hAnd a (-1)) a
    theorem UInt16.and_neg_one {a : UInt16} :
    Eq (HAnd.hAnd a (-1)) a
    theorem UInt32.and_neg_one {a : UInt32} :
    Eq (HAnd.hAnd a (-1)) a
    theorem UInt64.and_neg_one {a : UInt64} :
    Eq (HAnd.hAnd a (-1)) a
    theorem USize.and_neg_one {a : USize} :
    Eq (HAnd.hAnd a (-1)) a
    theorem UInt8.and_eq_neg_one_iff {a b : UInt8} :
    Iff (Eq (HAnd.hAnd a b) (-1)) (And (Eq a (-1)) (Eq b (-1)))
    theorem UInt16.and_eq_neg_one_iff {a b : UInt16} :
    Iff (Eq (HAnd.hAnd a b) (-1)) (And (Eq a (-1)) (Eq b (-1)))
    theorem UInt32.and_eq_neg_one_iff {a b : UInt32} :
    Iff (Eq (HAnd.hAnd a b) (-1)) (And (Eq a (-1)) (Eq b (-1)))
    theorem UInt64.and_eq_neg_one_iff {a b : UInt64} :
    Iff (Eq (HAnd.hAnd a b) (-1)) (And (Eq a (-1)) (Eq b (-1)))
    theorem USize.and_eq_neg_one_iff {a b : USize} :
    Iff (Eq (HAnd.hAnd a b) (-1)) (And (Eq a (-1)) (Eq b (-1)))
    theorem UInt8.xor_assoc (a b c : UInt8) :
    theorem UInt16.xor_assoc (a b c : UInt16) :
    theorem UInt32.xor_assoc (a b c : UInt32) :
    theorem UInt64.xor_assoc (a b c : UInt64) :
    theorem USize.xor_assoc (a b c : USize) :
    theorem UInt8.xor_comm (a b : UInt8) :
    Eq (HXor.hXor a b) (HXor.hXor b a)
    theorem UInt16.xor_comm (a b : UInt16) :
    Eq (HXor.hXor a b) (HXor.hXor b a)
    theorem UInt32.xor_comm (a b : UInt32) :
    Eq (HXor.hXor a b) (HXor.hXor b a)
    theorem UInt64.xor_comm (a b : UInt64) :
    Eq (HXor.hXor a b) (HXor.hXor b a)
    theorem USize.xor_comm (a b : USize) :
    Eq (HXor.hXor a b) (HXor.hXor b a)
    theorem UInt8.xor_self {a : UInt8} :
    Eq (HXor.hXor a a) 0
    theorem UInt16.xor_self {a : UInt16} :
    Eq (HXor.hXor a a) 0
    theorem UInt32.xor_self {a : UInt32} :
    Eq (HXor.hXor a a) 0
    theorem UInt64.xor_self {a : UInt64} :
    Eq (HXor.hXor a a) 0
    theorem USize.xor_self {a : USize} :
    Eq (HXor.hXor a a) 0
    theorem UInt8.xor_zero {a : UInt8} :
    Eq (HXor.hXor a 0) a
    theorem UInt16.xor_zero {a : UInt16} :
    Eq (HXor.hXor a 0) a
    theorem UInt32.xor_zero {a : UInt32} :
    Eq (HXor.hXor a 0) a
    theorem UInt64.xor_zero {a : UInt64} :
    Eq (HXor.hXor a 0) a
    theorem USize.xor_zero {a : USize} :
    Eq (HXor.hXor a 0) a
    theorem UInt8.zero_xor {a : UInt8} :
    Eq (HXor.hXor 0 a) a
    theorem UInt16.zero_xor {a : UInt16} :
    Eq (HXor.hXor 0 a) a
    theorem UInt32.zero_xor {a : UInt32} :
    Eq (HXor.hXor 0 a) a
    theorem UInt64.zero_xor {a : UInt64} :
    Eq (HXor.hXor 0 a) a
    theorem USize.zero_xor {a : USize} :
    Eq (HXor.hXor 0 a) a
    theorem UInt8.xor_eq_zero_iff {a b : UInt8} :
    Iff (Eq (HXor.hXor a b) 0) (Eq a b)
    theorem UInt16.xor_eq_zero_iff {a b : UInt16} :
    Iff (Eq (HXor.hXor a b) 0) (Eq a b)
    theorem UInt32.xor_eq_zero_iff {a b : UInt32} :
    Iff (Eq (HXor.hXor a b) 0) (Eq a b)
    theorem UInt64.xor_eq_zero_iff {a b : UInt64} :
    Iff (Eq (HXor.hXor a b) 0) (Eq a b)
    theorem USize.xor_eq_zero_iff {a b : USize} :
    Iff (Eq (HXor.hXor a b) 0) (Eq a b)
    theorem UInt8.xor_left_inj {a b : UInt8} (c : UInt8) :
    Iff (Eq (HXor.hXor a c) (HXor.hXor b c)) (Eq a b)
    theorem UInt16.xor_left_inj {a b : UInt16} (c : UInt16) :
    Iff (Eq (HXor.hXor a c) (HXor.hXor b c)) (Eq a b)
    theorem UInt32.xor_left_inj {a b : UInt32} (c : UInt32) :
    Iff (Eq (HXor.hXor a c) (HXor.hXor b c)) (Eq a b)
    theorem UInt64.xor_left_inj {a b : UInt64} (c : UInt64) :
    Iff (Eq (HXor.hXor a c) (HXor.hXor b c)) (Eq a b)
    theorem USize.xor_left_inj {a b : USize} (c : USize) :
    Iff (Eq (HXor.hXor a c) (HXor.hXor b c)) (Eq a b)
    theorem UInt8.xor_right_inj {a b : UInt8} (c : UInt8) :
    Iff (Eq (HXor.hXor c a) (HXor.hXor c b)) (Eq a b)
    theorem UInt16.xor_right_inj {a b : UInt16} (c : UInt16) :
    Iff (Eq (HXor.hXor c a) (HXor.hXor c b)) (Eq a b)
    theorem UInt32.xor_right_inj {a b : UInt32} (c : UInt32) :
    Iff (Eq (HXor.hXor c a) (HXor.hXor c b)) (Eq a b)
    theorem UInt64.xor_right_inj {a b : UInt64} (c : UInt64) :
    Iff (Eq (HXor.hXor c a) (HXor.hXor c b)) (Eq a b)
    theorem USize.xor_right_inj {a b : USize} (c : USize) :
    Iff (Eq (HXor.hXor c a) (HXor.hXor c b)) (Eq a b)
    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) :
    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) :
    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) :
    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) :
    theorem UInt8.and_le_left {a b : UInt8} :
    theorem USize.and_le_left {a b : USize} :
    theorem UInt8.left_le_or {a b : UInt8} :
    LE.le a (HOr.hOr a b)
    theorem UInt16.left_le_or {a b : UInt16} :
    LE.le a (HOr.hOr a b)
    theorem UInt32.left_le_or {a b : UInt32} :
    LE.le a (HOr.hOr a b)
    theorem UInt64.left_le_or {a b : UInt64} :
    LE.le a (HOr.hOr a b)
    theorem USize.left_le_or {a b : USize} :
    LE.le a (HOr.hOr a b)
    theorem UInt8.right_le_or {a b : UInt8} :
    LE.le b (HOr.hOr a b)
    theorem UInt16.right_le_or {a b : UInt16} :
    LE.le b (HOr.hOr a b)
    theorem UInt32.right_le_or {a b : UInt32} :
    LE.le b (HOr.hOr a b)
    theorem UInt64.right_le_or {a b : UInt64} :
    LE.le b (HOr.hOr a b)
    theorem USize.right_le_or {a b : USize} :
    LE.le b (HOr.hOr a b)