Documentation

Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Impl.Operations.Append

This module contains the implementation of a bitblaster for BitVec.append.

structure Std.Tactic.BVDecide.BVExpr.bitblast.AppendTarget {α : Type} [Hashable α] [DecidableEq α] (aig : Sat.AIG α) (combined : Nat) :
  • lw : Nat
  • rw : Nat
  • lhs : aig.RefVec self.lw
  • rhs : aig.RefVec self.rw
  • h : combined = self.rw + self.lw
Instances For
    def Std.Tactic.BVDecide.BVExpr.bitblast.blastAppend {α : Type} [Hashable α] [DecidableEq α] {newWidth : Nat} (aig : Sat.AIG α) (target : AppendTarget aig newWidth) :
    Equations
    Instances For