This module contains the verification of the bitblaster for BitVec.replicate
from Impl.Operations.Replicate
.
@[simp]
theorem
Std.Tactic.BVDecide.BVExpr.bitblast.denote_blastReplicate
{α : Type}
[Hashable α]
[DecidableEq α]
{newWidth : Nat}
(aig : Sat.AIG α)
(target : ReplicateTarget aig newWidth)
(assign : α → Bool)
(idx : Nat)
(hidx : idx < newWidth)
:
⟦assign, { aig := (blastReplicate aig target).aig, ref := (blastReplicate aig target).vec.get idx hidx }⟧ = ⟦assign, { aig := aig, ref := target.inner.get (idx % target.w) ⋯ }⟧