This module contains the implementation of a bitblaster for BitVec.clz
.
def
Std.Tactic.BVDecide.BVExpr.bitblast.blastClz
{α : Type}
[Hashable α]
[DecidableEq α]
{w : Nat}
(aig : Sat.AIG α)
(x : aig.RefVec w)
:
Equations
Instances For
@[irreducible]
def
Std.Tactic.BVDecide.BVExpr.bitblast.blastClz.go
{α : Type}
[Hashable α]
[DecidableEq α]
{w : Nat}
(aig : Sat.AIG α)
(x : aig.RefVec w)
(curr : Nat)
(acc : aig.RefVec w)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
instance
Std.Tactic.BVDecide.BVExpr.bitblast.instLawfulVecOperatorRefVecBlastClz
{α : Type}
[Hashable α]
[DecidableEq α]
:
Sat.AIG.LawfulVecOperator α Sat.AIG.RefVec fun {len : Nat} => blastClz