-
Couldn't load subscription status.
- Fork 243
Open
Description
open FStar.BV
// let _ : bv_t 128 = bv_zero
let int2bv_uext_64_128 (x1 : nat) :
Lemma (requires x1 < pow2 64) // (FStar.UInt.size x1 64))
(ensures bv_uext #64 #64 (int2bv #64 x1) == int2bv #128 x1) =
admit ()Gives:
* Error 276 at Basic.fst(10,0-14,10):
- Unexpected output from Z3:
"(error "line 11230 column 90: unknown function/constant BoxBitVec128")"
* Error 276 at Basic.fst(10,0-14,10):
- Unexpected output from Z3:
"(error "line 11284 column 90: unknown function/constant BoxBitVec128")"
* Error 276 at Basic.fst(10,0-14,10):
- Unexpected output from Z3:
"(error "line 11338 column 90: unknown function/constant BoxBitVec128")"
* Error 276 at Basic.fst(10,0-14,10):
- Unexpected output from Z3:
"(error "line 11394 column 90: unknown function/constant BoxBitVec128")"
* Error 276 at Basic.fst(10,0-14,10):
- Unexpected output from Z3:
"(error "line 11547 column 79: unknown function/constant BoxBitVec128")"
Verified module: Basic
5 errors were reported (see above)
Uncommenting the definition of that vector makes the encoding kick in.
Metadata
Metadata
Assignees
Labels
No labels