-
``` c++
void PrimeNumbers::FillBitVector(BitVector &bitVector, bool fillBit, size_t count)
{
assert(bitVector.empty());
bitVector.reserve(count);
for (size_t i = 0; i < count; ++i)
{
…
-
Example of misleading results:
```haskell
>>> 0xFF :: BitVector 8
1111_1111
>>> 1111_1111 :: BitVector 8
1100_0111
```
This could be fixed by pretending `0b`. Hypothetical new situation:
…
-
I want to try running the solvers on a problem I have, but I need either array or bitvector that is more than 64 bits. Is any of the solvers support either of these features? Enumeration solver suppor…
-
When experimenting with encoding set as bitvectors as `Nat`s, which seems like it should be rather efficient, I noticed that processing the file in VSCode was quick enough, but `lake build` would take…
-
It would be interesting to have additional arguments in the `trocq` tactic to provide guidance and tell Trocq which terms must change, and which must not. It would for example allow for several parame…
-
Hello,
I'm trying to work with SMTCoq (coq 8.18.0, cvc4 1.6) and this example puzzles me:
```coq
Require Import ZArith.
From SMTCoq Require Import SMTCoq BVList.
Import BITVECTOR_LIST.
Local…
-
I have a fairly complex proof that will involve lots of rewriting, and am encountering some issues. Here's a stripped-down example illustrating one of them.
In the context of this Cryptol
…
-
```haskell
{-# LANGUAGE UndecidableInstances #-}
module Issue where
import Clash.Prelude
type family Width a where
Width a = BitSize a
topEntity :: BitVector (Width Bool) -> ()
topEnt…
-
Type families are a hack. I would like to make them more elegant.
I want to define a class `Family` which expects that inheriting classes will have inner classes `Bit` and `BitVector`, then automa…
-
Currently the bitvectors in succinct are represented by `Data.Vector.Unboxed` `Vector`s. Allowing bitvectors of any `Vector` type would, among other things, enable easy disk backing of succinct struct…