Equations
- One or more equations did not get rendered due to their size.
theorem
UInt8.upwardEnumerableLE_ofBitVec
{x y : BitVec 8}
:
Std.PRange.UpwardEnumerable.LE { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LE x y
theorem
UInt8.upwardEnumerableLT_ofBitVec
{x y : BitVec 8}
:
Std.PRange.UpwardEnumerable.LT { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LT x y
Equations
- UInt8.instRangeSizeClosed = { size := fun (bound : Std.PRange.Bound Std.PRange.BoundShape.closed UInt8) (a : UInt8) => UInt8.toNat bound + 1 - a.toNat }
theorem
UInt8.rangeSizeSize_eq_toBitVec
{bound : Std.PRange.Bound Std.PRange.BoundShape.closed UInt8}
{x : BitVec 8}
:
Equations
- One or more equations did not get rendered due to their size.
theorem
UInt16.upwardEnumerableLE_ofBitVec
{x y : BitVec 16}
:
Std.PRange.UpwardEnumerable.LE { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LE x y
theorem
UInt16.upwardEnumerableLT_ofBitVec
{x y : BitVec 16}
:
Std.PRange.UpwardEnumerable.LT { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LT x y
Equations
- UInt16.instRangeSizeClosed = { size := fun (bound : Std.PRange.Bound Std.PRange.BoundShape.closed UInt16) (a : UInt16) => UInt16.toNat bound + 1 - a.toNat }
theorem
UInt16.rangeSizeSize_eq_toBitVec
{bound : Std.PRange.Bound Std.PRange.BoundShape.closed UInt16}
{x : BitVec 16}
:
Equations
- One or more equations did not get rendered due to their size.
theorem
UInt32.upwardEnumerableLE_ofBitVec
{x y : BitVec 32}
:
Std.PRange.UpwardEnumerable.LE { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LE x y
theorem
UInt32.upwardEnumerableLT_ofBitVec
{x y : BitVec 32}
:
Std.PRange.UpwardEnumerable.LT { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LT x y
Equations
- UInt32.instRangeSizeClosed = { size := fun (bound : Std.PRange.Bound Std.PRange.BoundShape.closed UInt32) (a : UInt32) => UInt32.toNat bound + 1 - a.toNat }
theorem
UInt32.rangeSizeSize_eq_toBitVec
{bound : Std.PRange.Bound Std.PRange.BoundShape.closed UInt32}
{x : BitVec 32}
:
Equations
- One or more equations did not get rendered due to their size.
theorem
UInt64.upwardEnumerableLE_ofBitVec
{x y : BitVec 64}
:
Std.PRange.UpwardEnumerable.LE { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LE x y
theorem
UInt64.upwardEnumerableLT_ofBitVec
{x y : BitVec 64}
:
Std.PRange.UpwardEnumerable.LT { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LT x y
Equations
- UInt64.instRangeSizeClosed = { size := fun (bound : Std.PRange.Bound Std.PRange.BoundShape.closed UInt64) (a : UInt64) => UInt64.toNat bound + 1 - a.toNat }
theorem
UInt64.rangeSizeSize_eq_toBitVec
{bound : Std.PRange.Bound Std.PRange.BoundShape.closed UInt64}
{x : BitVec 64}
:
Equations
- One or more equations did not get rendered due to their size.
theorem
USize.upwardEnumerableLE_ofBitVec
{x y : BitVec System.Platform.numBits}
:
Std.PRange.UpwardEnumerable.LE { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LE x y
theorem
USize.upwardEnumerableLT_ofBitVec
{x y : BitVec System.Platform.numBits}
:
Std.PRange.UpwardEnumerable.LT { toBitVec := x } { toBitVec := y } ↔ Std.PRange.UpwardEnumerable.LT x y
Equations
- USize.instRangeSizeClosed = { size := fun (bound : Std.PRange.Bound Std.PRange.BoundShape.closed USize) (a : USize) => USize.toNat bound + 1 - a.toNat }
theorem
USize.rangeSizeSize_eq_toBitVec
{bound : Std.PRange.Bound Std.PRange.BoundShape.closed USize}
{x : BitVec System.Platform.numBits}
: