Equations
- oneE5M10 = PackedFloat.ofBits 5 10 15360#16
Instances For
Equations
- twoE5M10 = PackedFloat.ofBits 5 10 16384#16
Instances For
Every floating point number converted to fixed point form, is an exact floating point number.
theorem
FP16_isExactFloat_round_toEFixed
(a : EFixedPoint 42 24)
(m : RoundingMode)
(ha : isExactFloat 5 10 a = true)
:
If a fixed point number is an exact floating point number, then converting to floating point and back should not change the denotation.
theorem
FP16_round_leftinv_toEFixed
(x : PackedFloat 5 10)
(mode : RoundingMode)
(hx : ¬x.isNaN = true)
:
Fixed -> Float rounding is left inverse to Float -> Fixed conversion
theorem
FP16_add_zero_is_id
(a : PackedFloat 5 10)
(m : RoundingMode)
(ha : ¬a.isNaN = true ∧ ¬a.isZero = true)
:
theorem
FP16_e_add_monotone
(m : RoundingMode)
(a b c : EFixedPoint 42 24)
(hc : c.state = State.Number)
:
theorem
FP16_add_monotone
(a b c : PackedFloat 5 10)
(m : RoundingMode)
(hc : c.isNormOrSubnorm = true)
:
NOTE: bv_decide SAT solver times out on this theorem.