Skip to main content
Springer logoLink to Springer
. 2020 May 22;65(1):125–154. doi: 10.1007/s10817-020-09560-1

Building Strategies into QBF Proofs

Olaf Beyersdorff 1,, Joshua Blinkhorn 1, Meena Mahajan 2
PMCID: PMC7808293  PMID: 33487785

Abstract

Strategy extraction is of great importance for quantified Boolean formulas (QBF), both in solving and proof complexity. So far in the QBF literature, strategy extraction has been algorithmically performed from proofs. Here we devise the first QBF system where (partial) strategies are built into the proof and are piecewise constructed by simple operations along with the derivation. This has several advantages: (1) lines of our calculus have a clear semantic meaning as they are accompanied by semantic objects; (2) partial strategies are represented succinctly (in contrast to some previous approaches); (3) our calculus has strategy extraction by design; and (4) the partial strategies allow new sound inference steps which are disallowed in previous central QBF calculi such as Q-Resolution and long-distance Q-Resolution. The last item (4) allows us to show an exponential separation between our new system and the previously studied reductionless long-distance resolution calculus. Our approach also naturally lifts to dependency QBFs (DQBF), where it yields the first sound and complete CDCL-style calculus for DQBF, thus opening future avenues into CDCL-based DQBF solving.

Keywords: QBF, DQBF, Resolution, Proof complexity

Introduction

Proof complexity investigates the resources for proving logical theorems, focussing foremost on the minimal size of proofs needed in a particular calculus. Since its inception the field has enjoyed strong connections to computational complexity (cf. [17, 20]) and to first-order logic [19, 38]).

During the past decade, proof complexity has emerged as a key tool to model and analyse advances in the algorithmic handling of hard problems such as SAT and beyond. While traditionally perceived as a computationally hard problem, SAT solvers have been enormously successful in tackling huge industrial instances [42, 56] and hard combinatorial problems [32]. As each run of a solver on an unsatisfiable formula can be understood as a proof of unsatisfiability, each solver implicitly defines a proof system. This connection turns proof complexity into the main theoretical approach towards understanding the power and limitations of solving, with bounds on proof size directly corresponding to bounds on solver running time [17, 43].

The algorithmic success story of solving has not stopped at SAT, but is currently extending to even more computationally complex problems such as quantified Boolean formulas (QBF), which is PSPACE complete, and dependency QBFs (DQBF), which is even NEXP complete [1]. While quantification does not increase expressivity, (D)QBFs can encode many problems far more succinctly, including application domains such as automated planning [18, 22], verification [6, 41], synthesis [24, 40] and ontologies [37].

The past 15 years have seen huge advances in QBF solving. While some of the main innovations in SAT solving, including the development of conflict-driven clause learning (CDCL), revolutionised SAT in the late 1990s [53], this development in QBF is happening now. Consequently, QBF proof complexity has received considerable attention in recent years.

Compared with QBF, solving in DQBF [26] is at its very beginnings, both in implementations (2018 was the first year that saw a DQBF track in the QBF competition [48]) as well as in its accompanying theory [52].

Strategy extraction is one of the distinctive features of QBF and DQBF, manifest in both solving [5, 49] and proof complexity. For solving it guarantees that together with the true/false answer the solver can produce a model (or countermodel) of the (D)QBF. This is an important step in the solving workflow, since a model (or countermodel) may encode a solution (or a counterexample) to the given problem. For example, a model for a QBF encoding a synthesis problem defines an implementation meeting the desired specification [31]. Determining truth merely implies the existence of such a system.

On the proof complexity side, this implies that proof calculi modelling QBF solving should allow strategy extraction in the sense that from a refutation of a false QBF, a countermodel of the QBF can be efficiently constructed. This feature—without analogue in the propositional domain—enables strong lower-bound techniques in QBF proof complexity [9, 11, 12], exploiting the fact that formulas requiring hard strategies cannot have short proofs in calculi with efficient strategy extraction.

As in SAT versus propositional proof complexity, one of the prime challenges in QBF and DQBF is to create compelling proof-theoretic models that capture central features of (D)QBF solving and at the same time remain amenable to a proof-theoretic analysis. While there exist several orthogonal approaches in QBF solving with quite different associated proof calculi, we will focus here on the paradigm of quantified conflict-driven constraint learning (QCDCL) [59]. An interesting feature of QCDCL is that it combines conflict learning with solution learning. Whereas a CDCL SAT solver can terminate upon finding a single solution (i.e. a satisfying assignment), a QCDCL QBF solver will repeatedly learn and manipulate solutions, aiming to determine the truth of the input QBF.1 Meanwhile, the solver also employs conflict learning, aiming to determine falsity. Here we focus on the conflict learning side. Proof-theoretically its most basic model is Q-Resolution [35], which as in propositional resolution operates on clauses (of prenex QBFs).

Q-Resolution (Q-Res) uses the resolution rule of propositional resolution and augments this with a universal reduction rule that allows to eliminate universal variables from clauses. Combining these two rules requires some technical care: without any side-conditions the two rules result in an unsound system. Typically this is circumvented by prohibiting the derivation of universal tautologies. It was noted early on that in solving this is needlessly prohibitive [59] and universal tautologies can be permitted under certain side-conditions. Later formalised as the proof system long-distance Q-Resolution (LD-Q-Res) [3], it was even shown that LD-Q-Res exponentially shortens proofs in comparison to Q-Res [23], thus demonstrating the appeal of the approach for solving. In fact, when enabling long-distance steps in QBF solving, universal reduction is not strictly needed and this reductionless approach was adopted in the QBF solver GhostQ [36]. To model this solving paradigm, Bjørner, Janota, and Klieber [15] introduced the calculus of reductionless LD-Q-Res.

The interplay between long-distance resolution and universal reduction steps becomes even more intriguing in DQBF. In [2] it was shown that lifting Q-Res (using the rules of resolution and universal reduction) to DQBF results in an incomplete proof system, whereas lifting LD-Q-Res (using long-distance resolution steps together with universal reduction) becomes unsound [13].

Naturally, the intriguing question of why and how deriving ‘universal tautologies’ in long-distance steps might help solving has attracted attention among theoreticians and practitioners alike. Instead of a universal tautology uu¯, most formalisations of long-distance resolution actually use the concept of a ‘merged’ literal u. While it is clear (and implicit in the literature) that merged literals u correspond to partial strategies for u rather than universal tautologies, a formal semantic account of long-distance steps (and stronger calculi using merging [12]) was only recently given by Suda and Gleiss [54], where partial strategies are constructed for each individual proof inference. However, as already noted in [54], the models considered in [54] fail to have efficient strategy extraction in the sense that the constructed (partial) strategies may need exponential-size representations.

Our contributions

A. The new calculus of Merge Resolution. Starting from the reductionless LD-Q-Res system of [15] and its role of modelling QCDCL solving, we develop a new calculus that we call Merge Resolution (M-Res). Like reductionless LD-Q-Res, the system M-Res only uses a resolution rule and does not permit universal reduction steps. Reductionless LD-Q-Res and M-Res are therefore both refutational calculi that finish as soon as they derive a purely universal clause.

As the prime novel feature of M-Res we build partial strategies into proofs. We achieve this by computing explicit representations of strategies in a variant of binary decision diagrams (called merge maps here), which are updated and refined at each proof step by simple operations. These merge maps are part of the proof. As a consequence, M-Res has efficient strategy extraction by design.

This is in contrast to all previous existing QBF calculi in the literature, where strategies are algorithmically constructed from proofs. In particular, this also applies to the approaches taken in [23, 54] for LD-Q-Res and in [15] for reductionless LD-Q-Res. But also the choice of our representation as merge maps matters: as [15, 54] both represent (partial) strategies as trees, the constructed strategies may grow exponentially in the proof size, thus losing the property of efficient strategy extraction desired for practice. In contrast, in our model merge maps are always linear in the size of the clause derivations.

B. Exponential separation of M-Res from reductionless LD-Q-Res. Including merge maps explicitly into proofs also has another far-reaching advantage: it allows resolution steps not only forbidden in Q-Res, but even disallowed in LD-Q-Res. In a nutshell, LD-Q-Res allows resolution steps only when universal variables quantified left of the pivot have constant and equal strategies in both parent clauses. In M-Res we have explicit representations of strategies and thus can allow resolution steps as long as the strategies in both parent clauses are isomorphic to each other, a property that we can check efficiently for merge maps.

This last mentioned advantage of allowing resolution steps in M-Res forbidden in (reductionless) LD-Q-Res manifests in shorter proofs. We show this by explicitly giving an example of a family of QBFs that admit linear-size proofs in M-Res (Theorem 29), but require exponential size in reductionless LD-Q-Res (Theorem 28). The separating formulas are a variant of the equality formulas introduced in [9]. While the original formulas from [9] are hard for Q-Res, but easy in LD-Q-Res, we here consider a ‘squared’ version, for which we naturally use resolution steps for clauses with associated non-constant winning strategies, allowed in M-Res, but forbidden in LD-Q-Res.

This demonstrates that M-Res is exponentially stronger than reductionless LD-Q-Res, thus also pointing towards potential improvements in QCDCL solving. While the simulation of reductionless LD-Q-Res by M-Res is almost immediate and also the upper bound in M-Res is comparatively straightforward, the lower bound is a technically involved argument specifically tailored towards the squared equality formulas.

C. A sound and complete CDCL-style calculus for DQBF. As our final contribution we show that the new QBF system of M-Res naturally lifts to a sound and complete calculus for DQBF. As shown in [2], the lifting of Q-Res to DQBF is incomplete, whereas the combination of universal reduction and long-distance steps presents soundness issues, both in DQBF [13] as well as in the related framework of dependency schemes [7, 8].

Here we show that our framework of M-Res overcomes both these soundness and completeness issues and therefore has exactly the right strength for a natural DQBF resolution calculus. In fact, it is the first DQBF CDCL-style system in the literature2 and as such paves the way towards CDCL-style solving in DQBF. Again, by design our DQBF system has efficient strategy extraction.

Preliminaries

Propositional logic Let Z be a countable set of Boolean variables. A literal is a Boolean variable zZ or its negation z¯, a clause is a set of literals, and a CNF is a set of clauses. For a literal l, we define var(l):=z if l=z or l=z¯; for a clause C, we define vars(C):={var(l):lC}; for a CNF ϕ we define vars(ϕ):=Cϕvars(C).

An assignment to a set ZZ of Boolean variables is a function ρ:Z{0,1}, conventionally represented as a set of literals in which z (resp. z¯) represents the assignment z1 (resp. z0). The set of all assignments to Z is denoted Z. Given a subset ZZ, ρZ is the restriction of ρ to Z. The CNF ϕ[ρ] is obtained from ϕ by removing any clause containing a literal in ρ, and removing the negated literals {l¯:lρ} from the remaining clauses. We say that ρ falsifies ϕ if ϕ[ρ] contains the empty clause, and that ϕ is unsatisfiable if it is falsified by each ρZ.

Given two clauses R1 and R2 and a literal l such that lR1 and l¯R2, we define the resolvent res(R1,R2,l):=(R1\{l})(R2\{l¯}). (Note that res(R1,R2,l)=res(R2,R1,l¯).) A resolution refutation of a CNF ϕ is a sequence C1,,Ck of clauses in which Ck is the empty clause and, for each i[k], either (a) Ciϕ or (b) Ci=res(Ca,Cb,z) for some a,b<i and zvars(ϕ).

Quantified Boolean formulas A quantified Boolean formula (QBF) in prenex conjunctive normal form (PCNF) is denoted Φ:=Q·ϕ, where (a) Q:=Q1Z1QnZn is the quantifier prefix, in which the ZiZ are pairwise disjoint finite sets of Boolean variables, Qi{,} for each i[n], and QiQi+1 for each i[n-1], and (b) the matrix ϕ is a CNF over vars(Φ):=i=1nZi.

The existential (resp. universal) variables of Φ, typically denoted X (resp. U), is the set obtained as the union of the Zi for which Qi= (resp. Qi=). The prefix Q defines a binary relation <Q on vars(Φ), such that z<Qz holds iff zZi, zZj, and i<j, in which case we say that z is right of z and z is left of z. For each uU, we define LQ(u):={xX:x<Qu}, i.e. the existential variables left of u.

QBF semantics Semantics for QBFs is neatly described by the two-player evaluation game. Over the course of a game, the variables of a QBF Q·ϕ are assigned 0/1 values in the order of the prefix, with the -player (-player) choosing the values for the existential (universal) variables. When the game concludes, the players have constructed a total assignment ρ to the variables. The -player wins iff ρ falsifies ϕ.

A strategy dictates how the -player should respond to every possible move of the -player. A strategy h for a QBF Φ is a set {hu:uU} of functions hu:LQ(u){u,u¯}. Additionally h is winning if, for each αX, the restriction of ϕ by α{hu(αLQ(u)):uU} contains the empty clause. We use the terms ‘winning strategy’ and ‘countermodel’ interchangeably. A QBF is called false if it has a countermodel, and true if it does not.

A partial strategy for a universal variable u is a function from some subset of LQ(u) into {u,u¯}.

QBF proof systems We deal with line-based refutational QBF systems that typically employ axioms and inference rules to prove the falsity of QBFs. We say that P is complete if there exists a P refutation of every false QBF, sound if there exists no P refutation of any true QBF. We call P a proof system if it is sound, complete, and polynomial-time checkable. Given two QBF proof systems P1 and P2, P1 p-simulates P2 if there exists a polynomial-time procedure that takes a P2-refutation and outputs a P1-refutation of the same QBF [20].

Reductionless long-distance Q-Resolution

In this section we recall the definition of reductionless LD-Q-Res, prove that it is refutationally complete, and demonstrate that it does not have polynomial-time strategy extraction in either of the computational models of [15, 54]. The system appeared first in [15, Fig. 1], where it was referred to as Qw-resolution.

Definition 1

(reductionless LD-Q-Res [15]) In reductionless LD-Q-Res, a derivation from a QBF Φ:=Q·ϕ is a sequence π:=C1,,Ck of clauses in which at least one of (a) or (b) holds for each i[k]:

  1. Axiom. Ci is a clause from the matrix ϕ;

  2. Long-distance resolution. There exist integers a,b<i and an existential pivot xX such that Ci=res(Ca,Cb,x) and, for each uvars(Ca)vars(Cb), if u<Qx, then {u,u¯}Ci.

The final clause Ck is the conclusion of π, and π is a refutation of Φ iff Ck contains no existential variables.

A pair of complementary universal literals {u,u¯} appearing in a clause is referred to singly as a merged literal. It is clear from a wealth of literature3 that merged literals are ‘placeholders’ for partial strategies, the exact representation left implicit in the structure of the derivation.

We illustrate the rules of the calculus by showing that the equality formulas [9] have linear-size refutations.

Definition 2

(equality formulas [9]) The equality family is the QBF family whose nth instance has the prefix {x1,,xn}{u1,,un}{t1,,tn} and the matrix consisting of the clauses {xi,ui,ti},{x¯i,u¯i,ti} for i[n], and {t¯1,,t¯n}.

Example 3

We construct linear-size reductionless LD-Q-Res refutations in two stages. First, resolve each pair {xi,ui,ti}, {x¯i,u¯i,ti} of clauses over pivot xi to obtain Ci:={ui,u¯i,ti}. Note that it is allowed to introduce the merged literal {ui,u¯i} since variable ui is right of the pivot xi. Second, resolve the Ci successively against the long clause {t¯1,,t¯n} over pivot ti, to obtain a full set of merged literals C:={ui,u¯i:i[n]}. Here, even though ui is left of the pivot ti, the appearance of the merged literal {ui,ui¯} in the resolvent is allowed, since variable ui is absent from one of the antecedents. The derivation is a refutation since the conclusion C contains no existential literals.

We now show that this calculus is indeed complete. Given a false QBF Φ with a countermodel h, we construct a canonical reductionless LD-Q-Res refutation based on the ‘full binary tree’ representation of a countermodel [51]. For each αX, there exists some Cα in the matrix falsified by αh(α). The set of all such Cα may be successively resolved over existential pivots in reverse prefix order, finally producing a clause containing no existentials. Merged literals never block resolution steps in this construction, as they only ever appear to the right of the pivot variable.

Example 4

Consider the QBF with the prefix {x}{u}{y}{v} and the matrix consisting of the clauses

{x,u,y,v},{x,u,y¯,v¯},{x¯,u¯,y,v},{x¯,u¯,y¯,v¯}.

It is easy to see that the unique countermodel for this QBF essentially sets u and v equal to x and y, respectively. Formally, the countermodel consists of the functions hu and hv, where hu(α)(u)=α(x) and hv(β)(v)=β(y), for each α{x} and β{x,y}.

Figure 1 shows the full binary tree depiction of this countermodel and its associated reductionless LD-Q-Res refutation. Notice that each path from root to leaf in the countermodel tree specifies a total assignment that falsifies the corresponding axiom clause. Notice also that the existential resolution pivots on each path from an axiom to the conclusion occur in reverse prefix order, matching the pattern of the full binary tree countermodel. The prefix order inherent to the countermodel tree also ensures that each long-distance resolution step is valid.

Fig. 1.

Fig. 1

The full binary tree depiction of a countermodel and its associated reductionless LD-Q-Res refutation

Lemma 5

Every false QBF has a reductionless LD-Q-Res refutation.

Proof

Let Φ:=Q·ϕ be a false QBF with countermodel h. Let {x1,,xn} denote the existential variables of Φ in prefix order; that is, for each i,j[n] with i<j, xi is not right of xj. Let α1,,α2n define the natural lexicographic ordering of the total assignments to X, as in

graphic file with name 10817_2020_9560_Equ23_HTML.gif

We define a sequence π:=πnπ0 in which each πi:=C1i,,C2ii, and the clauses Cji are defined recursively as follows: For j[2n], Cjn is any clause in ϕ falsified by αjh(αj) (at least one such clause exists by definition of countermodel); for i[n] and j[2i-1], Cji-1:=res(C2j-1i,C2ji,xi) if this resolvent exists, otherwise

Cji-1:=C2j-1i,ifxiC2j-1i,C2ji,ifx¯iC2ji.

It is readily verified by downwards induction on i[n] that each Cji contains no complementary universal literals in variables left of xi. Moreover, it is easy to see that the conclusion C10 contains no existential literals. Removing duplicate clauses from π produces a reductionless LD-Q-Res refutation of Φ.

Soundness and polynomial-time checkability of reductionless LD-Q-Res are immediate, as the system uses a subset of the rules of the classical long-distance Q-resolution proof system [3].

The computational model of Bjørner et al. [15]. In tandem with reductionless LD-Q-Res, the authors of [15] introduced a computational model based on tree-like branching programs. The model is used to explicitly construct the partial strategies represented implicitly by merged literals.

We demonstrate that tree-like branching programs constructed in this way cannot represent strategies efficiently; that is, the system does not have polynomial-time strategy extraction in the associated model (even for partial strategies). The following example shows a linear-size derivation whose explicit strategy grows exponentially large.

Example 6

Consider the following proof fragment, in reductionless LD-Q-Res, with a prefix vxwuyz. Alongside each proof line is the strategy for the universal variable u, as built by the Build function in [15]. In a nutshell, Build traverses the subderivation of the current step, and represents the pattern of merges on u as a tree-like branching program that queries the (existential) resolution pivots.

Line Obtained as Clause Strategy as built in [15]
C1 axiom {w,x,u} 0
C2 axiom {w¯,x,u¯} 1
C3 res(C1,C2,w) {x,u,u¯} w?1:0
C4 axiom {x¯,u,y} 0
C5 res(C3,C4,x) {u,u¯,y} x?0:[w?1:0]
C6 axiom {v,y¯}
C7 res(C5,C6,y) {v,u,u¯} x?0:[w?1:0]
C8 axiom {x¯,z}
C9 res(C3,C8,x) {u,u¯,z} w?1:0
C10 axiom {v¯,z¯}
C11 res(C9,C10,z) {v¯,u,u¯} w?1:0
C12 res(C7,C11,v) {u,u¯} v?(w?1:0):(x?0:[w?1:0])

Observe that the final strategy at line 12 represents the strategy corresponding to line 3 twice. By nesting such a proof fragment from lines C3 to C12 with fresh copies of the existential variables (vxyz) k times, we can construct a reductionless LD-Q-Res proof fragment with O(k) lines, where the strategy built by the Build function from [15] has size exponential in k.

The computational model of Suda and Gleiss [54].  The authors of [54] proposed a model of partial strategies based on so-called policies (a policy is a set of assignments specifying an ordered decision tree.) They noted that the equality formulas have linear-size refutations in the strong QBF system IRM-calc [12], whereas policies witnessing their falsity must be exponentially large, therefore IRM-calc does not admit polynomial-time strategy in policies. The same is true for reductionless LD-Q-Res, since Example 3 shows that the equality formulas also have linear-size refutations there.

The computational model of policies is not even suitable for strategy extraction in the weak system level-ordered Q-Res [34].4 Versions of the equality formulas in which the prefix is rearranged (x1u1t1xnuntn) have linear-size level-ordered Q-Res refutations, whereas winning strategies represented as policies must be large. The argument is the same as for the equality formulas [54], and derives from the implicit use of tree-like structures.

That neither model is suitable for efficient strategy extraction shows that using either inside the derivation would result in an artificial, exponential size blow-up. The root of the issue is tree-like models versus DAG-like proofs. The DAG-like computational model that we introduce in the following section is tightly knitted to the refutation, yielding linear-time strategy extraction for free.

Merge resolution

In this section we introduce Merge Resolution (M-Res, Sect. 4.2), and prove that it is sound and complete for QBF (Sect. 4.3). The salient feature of M-Res is the built-in partial strategies, represented as merge maps. Given the problems with the computational models of [15, 54], the principal technical challenge is to find a suitable way to define and combine partial strategies devoid of an artificial proof-size inflation.

Merge maps

Our computational model A merge map is a branching program that queries a set of existential variables and outputs an assignment to some universal variable, i.e. a literal in {u,u¯,}, where stands for ‘no assignment’. As we intend to tie the DAG structure of the merge maps to the DAG structure of the proof, we will label query nodes with natural numbers based on the proof line indexing (we elaborate on this later). Hence, from a technical standpoint it makes sense to define a merge map as a function from the index set of its nodes.

Definition 7

(merge map) A merge map M for a Boolean variable u over a finite set X of Boolean variables is a function from a finite set N of natural numbers satisfying, for each iN, either M(i){u,u¯,} or M(i)X×N<i×N<i, where N<i:={iN:i<i}.

A triple of the form (x,a,b)X×N<i×N<i represents the instruction ‘if x=0 then goto a else goto b’, whereas the literals {u,u¯,} represent output values. The exact computation is formalised below.

Definition 8

(computed function) Let M be a merge map for u over X with domain N. The function computed by M is the function

h:X{u,u¯,}

mapping αX to the output of the following algorithm:

  1. i:=max(N)

  2. whileM(i){u,u¯,}

  3. (x,a,b):=M(i)

  4. ifx¯αtheni:=aelsei:=b

  5. returnM(i)

We depict merge maps pictorially as DAGs. The nodes are the domain elements, and the leaf nodes as well as the directed edges are labelled by literals. In a merge map M, if M(i) is a literal l, then node i is labeled l. If M(i)=(x,a,b), then the DAG has the edge ia labeled x¯ and the edge ib labeled x. The DAG naturally describes a deterministic branching program computing a Boolean function.

Figure 2 shows a merge map represented as a function, and its corresponding depiction as a branching program.

Fig. 2.

Fig. 2

Function and branching program representations of a merge map M

Relations Merge Resolution uses two relations to determine preconditions for the binary operations. Firstly, we give M-Res the power to identify merge maps with equivalent representations, up to indexing. We term equivalent representations ‘isomorphic’.

Definition 9

(isomorphism) Two merge maps M1 and M2 for u over X with domains N1 and N2 are isomorphic (written M1M2) iff there exists a bijection f:N1N2 such that the following hold for each iN1:

  1. if M1(i) is a literal in {u,u¯,} then M2(f(i))=M1(i);

  2. if M1(i) is the triple (xab) then M2(f(i))=(x,f(a),f(b)).

Proposition 10

Any two isomorphic merge maps compute the same function.

Proof

Let M1 and M2 be merge maps, let f be a bijection satisfying the properties of Definition 9, and let idom(M1). The computation of M2(i) as in Definition 8 is identical to that of M1, except that each natural number adom(M1) is replaced with f(a). The proposition follows.

Our second relation, consistency, simply identifies whether or not two merge maps agree on the intersection of their domains.

Definition 11

(consistency) Two merge maps M1 and M2 for u over X with domains N1 and N2 are consistent (written M1M2) iff M1(i)=M2(i) for each iN1N2.

Example 12

For the merge maps depicted in Fig. 3, isomorphism and consistency (or lack thereof) are as given in the table below.

Fig. 3.

Fig. 3

Relations on merge maps

Relation Isomorphic Not isomorphic
Consistent AC; AC BD; BD
Not consistent A⋈̸B; AB C⋈̸D; CD

It is easy to see that both relations can be computed in time polynomial in max(N1N2). (To check isomorphism, step through the two merge maps starting from their maximal domain elements N1,N2. Using memoization, iteratively build the bijection-witnessing isomorphism. Any suitable data structure that allows efficient insertion and search can be used for this. To check consistency, construct the two domains—again, using an appropriate data structure, and check that the instructions at common line numbers match.)

Operations M-Res uses two binary operations to build merge maps for the resolvent based on those of the antecedents. We define the operations and give some intuition on their role in M-Res. Concrete examples follow the definition of the system in the next subsection.

The select operation identifies equivalent merge maps by means of the isomorphism relation. It also allows a trivial merge map to be discarded; we call a merge map trivial iff it is isomorphic to 1. (The operation is undefined if the merge maps are neither isomorphic nor do they contain a trivial map.)

Definition 13

(select) Let M1 and M2 be merge maps for which M1M2 or one of M1,M2 is trivial. Then select(M1,M2):=M2 if M1 is trivial, and select(M1,M2):=M1 otherwise.

The merge operation allows two consistent merge maps to be combined as the children of a fresh query node. Antecedent maps are only ever merged for universal variables right of the pivot x. The inclusion of a natural number n allows the new query node to be identified with the resolvent, via its index in the proof sequence. In this way, query nodes are shared between later merge maps, rather than being duplicated; the result is a DAG-like structure which faithfully follows that of the derivation.

Definition 14

(merge) Let M1 and M2 be consistent merge maps for u over X with domains N1 and N2, let n>max(N1N2) be a natural number, and let xX. Then merge(M1,M2,n,x) is the function from N1N2{n} defined by

merge(M1,M2,n,x)(i):=(x,max(N1),max(N2))ifi=n,M1(i)ifiN1,M2(i)ifiN2\N1.

Example 15

In Fig. 3, we have select(A,B)=select(A,C)=A. Also, merge(D,B,6,v) gives the merge map from Fig. 2.

Definition of M-Res

We are now ready to put down the rules of Merge Resolution. Given a non-tautological clause C and a Boolean variable u, the falsifying u-literal for C is l¯ if there is a literal lC with var(l)=u, and otherwise.

Definition 16

(merge resolution) Let Φ:=Q·ϕ be a QBF with existential variables X and universal variables U. A merge resolution (M-Res) derivation of Lk from Φ is a sequence π:=L1,,Lk of lines Li:=(Ci,{Miu:uU}) in which at least one of the following holds for each i[k]:

  1. Axiom. There exists a clause in Cϕ such that Ci is the existential subclause of C, and, for each uU, Miu is the merge map for u over LQ(u) with domain {i} mapping i to the falsifying u-literal for C;

  2. Resolution. There exist integers a,b<i and an existential pivot xX such that Ci=res(Ca,Cb,x) and, for each uU, either
    • (i)
      Miu=select(Mau,Mbu), or
    • (ii)
      x<Qu and Miu=merge(Mau,Mbu,i,x).

The final line Lk is the conclusion of π, and π is a refutation of Φ iff Ck=. The size of π is |π|=k.

Note that the order of the indexes a and b in merge(Ma,Mb,i,x) matches that of res(Ca,Cb,x). This is why we interpret the triple (xab) as ‘if x=0 then goto a else goto b’. Using the conventional ‘if x=1’ entails swapping the order of the arguments Ma and Mb.

We illustrate the rules of M-Res with two examples. The first demonstrates that labelling branching nodes with proof-line indexes sidesteps the exponential blow-up in the computational model of [15].

Example 17

The reductionless LD-Q-Res proof fragment in Example 6 can be viewed as a proof in M-Res if we attach appropriate merge maps at each line.

Line Rule Ci Mi Query
L1 axiom {w,x} 1u¯
L2 axiom {w¯,x} 2u
L3 res(L1,L2,w) {x} merge(M1,M2,3,w) 3(w,1,2)
L4 axiom {x¯,y} 4u¯
L5 res(L3,L4,x) {y} merge(M3,M4,5,x) 5(x,3,4)
L6 axiom {v,y¯} 6
L7 res(L5,L6,y) {v} select(M5,M6)=M5
L8 axiom {x¯,z} 8
L9 res(L3,L8,x) {z} select(M3,M8)=M3
L10 axiom {v¯,z¯} 10
L11 res(L9,L10,z) {v¯} select(M9,M10)=
select(M3,M10)=M3
L12 res(L7,L11,v) {} merge(M7,M11,12,v) 12(v,5,3)
=merge(M5,M3,12,v)

In lines L7, L9 and L11, the use of select is allowed, since in each case one of the antecedent merge maps is trivial (i.e. isomorphic to 1). Notice that at line L7, we could also have chosen M7 to be merge(M5,M6,7,y); this would result in a larger merge map.

Now, consider the final merge map M12. The corresponding branching program has isolated nodes numbered 6, 8, and 10; these can be removed, giving the pruned merge map shown in Fig. 4. Notice how the size blow-up from Example 6 is avoided here; since M3 and M5 are consistent, node 12 simply points to both of them, and the shared part (that is, the branching program M3 containing nodes 1, 2, and 3) is represented just once.

Fig. 4.

Fig. 4

Function and branching program representations of M12 from Example 17

Our second example illustrates how the explicit representation of strategies, in tandem with the isomorphism relation, gives M-Res access to resolution steps that are disallowed in reductionless LD-Q-Res.

Example 18

Consider the following M-Res refutation of the QBF with prefix xut and clauses {x,u,t}, {x¯,u¯,t}, {x,u,t¯} and {x¯,u¯,t¯}.

Line Rule Ci Mi Query
L1 axiom {x,t} 1u¯
L2 axiom {x¯,t} 2u
L3 res(L1,L2,x) {t} merge(M1,M2,3,x) 3(x,1,2)
L4 axiom {x,t¯} 4u¯
L5 axiom {x¯,t¯} 5u
L6 res(L4,L5,x) {t¯} merge(M4,M5,6,x) 6(x,4,5)
L7 res(L3,L6,t) {} select(M3,M6)=M3

As shown in Fig. 5, M3 and M6 are isomorphic, so select(M3,M6) is defined and equal to M3. For this reason, the resolution of antecedents L3 and L6 into L7 is allowed, and the final merge map M7 is simply a copy of M3. The analogous resolution would be disallowed in reductionless LD-Q-Res because the pivot t is right of u, and the non-constant merge maps M3 and M6 would appear as merged literals {u,u¯} in the antecedent clauses.

Fig. 5.

Fig. 5

Functions and branching programs for merge maps M3 and M6 from Example 18

We conclude this subsection by showing that the number of lines really is the correct size measure for Merge Resolution. The justification lies in the fact that the domain of the merge map at line i is a subset of [i].

Proposition 19

Let (C1,{M1u:uU}),,(Ck,{Mku:uU}) be an M-Res refutation of Q·ϕ. For each uU, M1u,,Mnu are pairwise consistent merge maps for u over LQ(u) with max(dom(Miu))i for each i[n].

Proof

The claim follows straightforwardly from three observations: (1) each Miu introduces at most one node, which is labelled i; (2) if Li is an axiom, then each Miu is a merge map over LQ(u); (3) the merge operation is only applied when xLQ(u).

Soundness and completeness of M-Res

The soundness of M-Res comes down to the fact that the merge maps at a given line form a partial strategy for the input QBF, in the technical sense of [54]. This means that any total existential assignment that falsifies the clause Ci will falsify the matrix when extended by the output of the merge maps Miu. Our proof of soundness is an induction on the proof structure with exactly this invariant. At the conclusion, all existential assignments falsify the empty clause Ck, and hence the Mku compute a countermodel. A trivial corollary, then, is that M-Res has linear strategy extraction in merge maps. Our formal proof of soundness is preceded by a preliminary proposition.

Proposition 20

Let M1 and M2 be consistent merge maps for u over X with domains N1 and N2, let n>max(N1N2) be a natural number, let xX and let αX. Further, let h1,h2 and h be the functions computed by M1, M2 and merge(M1,M2,x,n). Then h(α)=h1(α) if x¯α, and h(α)=h2(α) if xα.

Proof

Let M:=merge(M1,M2,n,x), and suppose that x¯α. By Definition 14, M(n)=(x,max(N1),max(N2)) and M(i)=M1(i) for each iN1. Hence, the computation of h(α) from the second iteration of the while loop is identical to the computation of h1(α) from the first iteration, and it follows that h(α)=h1(α). Suppose instead that xα. By Definition 14, M(i)=M2(i) for each iN2\N1; by Definition 11, M1(i)=M2(i) for each iN1N2. Then M(i)=M2(i) for each iN2, and the proposition follows as in first case.

Lemma 21

Let (,{Mu:uU}) be the conclusion of an M-Res refutation of a QBF Φ. Then the functions computed by {Mu:uU} form a countermodel for Φ.

Proof

Let π:=L1,,Lk be an M-Res refutation of a QBF Φ:=Q·ϕ, where each Li=(Ci,{Miu:uU}). Further, for each i[k],

  • let αi:={l¯:lCi} be the smallest assignment falsifying Ci,

  • let Ai:={αX:Ciα=} be all assignments to X consistent with αi,

  • for each uU, let hiu be the function computed by Miu,

  • for each αAi, let liu(α):=hiu(proj(α,LQ(u))) and hi(α):={liu(α):uU}\{}.

(Note that Proposition 19 guarantees that each hiu is defined.) By induction on i[k], we show, for each αAi, that the restriction of ϕ by αhi(α) contains the empty clause. Since αk is the empty assignment, we have Ak=X. We therefore prove the lemma at the final step i=k, as we show that {hku:uU} is a countermodel for Φ.

For the base case i=1, let αA1. As L1 is introduced as an axiom, there exists a clause Cϕ such that C1 is the existential subclause of C, and each M1u is the merge map from {i} mapping i to the falsifying u-literal for C. Hence, for each uU, l1u(α) is the falsifying u-literal for C, so C[αh1(α)]=.

For the inductive step, let i2 and let αAi. The case where Li is introduced as an axiom is identical to the base case, so we assume that Li was derived by resolution. Then there exist integers a,b<i and an existential pivot xX such that Ci=res(Ca,Cb,x), and each uU satisfies either (i) Miu=select(Mau,Mbu), or (ii) xLQ(u), and Miu=merge(Mau,Mbu,i,x). Now, suppose on the one hand that x¯α, and let uU. If u satisfies (i) and Mau is non-trivial, then liu(α)=lau(α), and if u satisfies (ii) then liu(α)=lau(α) by Proposition 20. It follows that liulau only if lau=, and hence ha(α)hi(α). Since Ca{x}Ci, we have αAa, so the restriction of ϕ by αhi(α) contains the empty clause by the inductive hypothesis. Supposing, on the other hand, that xα, a similar argument shows that hb(α)hi(α). Note that, in this case, if u satisfies (i) and Mbu is non-trivial, then MauMbu and liu=lau=lbu by Proposition 10.

We show the completeness of M-Res via the p-simulation of reductionless LD-Q-Res. The simulation copies precisely the structure of the reductionless LD-Q-Res refutation, while replacing merged literals by merge maps in the natural way.

Theorem 22

M-Res p-simulates reductionless LD-Q-Res.

Proof

Let Φ:=Q·ϕ be a QBF with existential variables X and universal variables Y, and let π:=C1,,Ck be a reductionless LD-Q-Res refutation of Φ. We define a sequence π:=L1,,Ln, in which each Li:=(Ci,{Miu:uU}), and prove that it is an M-Res refutation of Φ.

For each i[k], we define Ci to be the existential subclause of Ci. For each uU, the merge maps are defined recursively as follows: If Ci is an axiom, Miu is defined as the merge map over LQ(u) with domain {i} mapping i to the falsifying u-literal for Ci (note that this covers the definition of M1u). If Ci is derived by resolution, say Ci=res(Ca,Cb,x) with a,b<i, then

Miu:=select(Mau,Mbu),ifselect(Mau,Mbu)isdefined,merge(Mau,Mbu,i,x),otherwise.

Now, by induction on i[k], we prove that, for each uU,

  1. if {u,u¯}Ci, then Miu is isomorphic to 1l, where l is the falsifying u-literal for Ci,

  2. Li can be derived from previous lines in π using an M-Res rule.

Both are established trivially when Ci is an axiom; hence it remains to show the inductive step in the case where Ci was derived by resolution. In this case Ci=res(Ca,Cb,x) for some a,b<i and some xX.

  1. Suppose that {u,u¯}Ci, and let li,la,lb be the falsifying u-literals for Ci,Ca,Cb. By definition of resolution, either (1) li=la=lb, or (2) exactly one of la,lb is trivial (lb, say), the other is equal to li. In the former case, Mau and Mbu are both isomorphic to 1li, by the inductive hypothesis; in the latter case, Mau is isomorphic to 1li and Mbu is trivial. Either way we get Miu=select(Mau,Mbu)=Mau, and the inductive step follows.

  2. By Proposition 19, for each uU, Mau and Mbu are consistent merge maps for u over LQ(u), so merge(Mau,Mbu,i,x) is defined for any case. Hence, if we can show that select(Mau,Mbu) is defined whenever u<Qx, then it is clear that Li can be derived by resolution from La and Lb. To that end, let u be left of x. If {u,u¯}Ci, then select(Mau,Mbu) is defined by (a). Otherwise, we must have uvars(Ca)vars(Cb), so the falsifying u-literal for one of Ca and Cb is By the inductive hypothesis, one of Mau and Mbu is trivial, and select(Mau,Mbu) is defined.

This completes the induction. Since Cn contains only universal variables, Ck is the empty clause, and π is a refutation.

With soundness and completeness established by Lemma 21 and Theorem 22, it remains to show that M-Res refutations can be checked in polynomial time. This is easy to see, since the isomorphism and consistency relations are computable efficiently.

Theorem 23

M-Res is a QBF proof system.

Proof complexity: merge resolution versus reductionless LD-Q-Res

In this section we exponentially separate M-Res from reductionless LD-Q-Res. The separating formulas are a kind of ‘squaring’ of the equality formulas from Definition 2.

Definition 24

(squared equality formulas) The squared equality family is the QBF family whose nth instance Inline graphic has the prefix

Q(n):={x1,y1,,xn,yn}{u1,v1,,un,vn}{ti,j:i,j[n]},

and the matrix Inline graphic consisting of the clauses

graphic file with name 10817_2020_9560_Equ24_HTML.gif

The only winning strategy for the universal player is to set ui=xi and vj=yj for each i,j[n]. At the final block, the existential player is faced with the full set of {ti,j} unit clauses, and to satisfy all of them is to falsify the square clause {t¯i,j:i,j[n]}. No other strategy can be winning, as it would fail to produce all n2 unit clauses.

Inline graphic lower bound for reductionless LD-Q-Res

We first give a formal definition of a refutation path; that is, a sequence of consecutive resolvents beginning with an axiom and ending at the conclusion.

Definition 25

(path) Let π be a reductionless LD-Q-Res refutation. A path from a clause C in π is a subsequence C1,,Ck of π in which:

  • C=C1 is an axiom of π;

  • Ck is the conclusion of π;

  • for each i[k-1], there exists a literal pi and a clause Ri occurring before Ci+1 in π such that Ci+1=res(Ci,Ri,pi).

The lower-bound proof is based upon two facts: (1) every total existential assignment corresponds to a path, all of whose clauses are consistent with the assignment (Lemma 26); (2) every path from the square clause contains a ‘wide’ clause containing either all the xi or all the yj variables (Lemma 27). It is then possible to deduce the existence of exponentially many wide clauses, i.e. by considering the set of assignments for which each xi=yi and each ti,j=0, all of whose corresponding paths begin at the square clause (proof of Theorem 28).

Lemma 26

Let π be a reductionless LD-Q-Res refutation of a QBF Φ, and let A be a clause with vars(A)=vars(Φ). Then there exists a path in π in which no existential literal outside of A occurs.

Proof

We describe a procedure that constructs a sequence P:=Ck,,C1 of clauses in reverse order as follows: To begin with, let the ‘current clause’ C1 be the conclusion of π. As soon as the current clause Ci is in an axiom, the procedure terminates. Whenever necessary, obtain Ci+1 as follows: find clauses R1 and R2 occurring before Ci in π and a literal pA such that Ci is res(R1,R2,p), and set Ci+1:=R1 as the current clause. P is clearly a path in π by construction. By induction one shows that the existential subclause of Ci is a subset of A, for each i[k]: The base case i=1 holds trivially since there are no existential literals in the conclusion C1 of π. For the inductive step, observe that Ci+1=C{p}, for some subset CCi and literal pA.

The second lemma is more technical, and its proof more involved. The proof works directly on the definition of path, the rules of reductionless LD-Q-Res, and the syntax of the squared equality formulas, to show the existence of the wide clause.

Lemma 27

Let n2, and let π be a reductionless LD-Q-Res refutation of Inline graphic. On each path from {t¯i,j:i,j[n]} in π, there occurs a clause C for which either {x1,,xn}vars(C) or {y1,,yn}vars(C).

Proof

Put X:={x1,,xn} and Y:={y1,,yn}. Call a clause R in π a p-resolvent if there exist earlier clauses R1 and R2 such that R=res(R1,R2,p).

Let P:=C1,,Ck be a path from {t¯i,j:i,j[n]} in π. With each Cl we associate an n×n matrix Ml in which Ml[i,j]:=1 if t¯i,jCi and Ml[i,j]:=0 otherwise. Let l be the least integer such that Ml has either a 0 in each row or a 0 in each column. Note that l2 since M1 has no zeros.

We prove the lemma by showing that either Xvars(Cl) or Yvars(Cl) must hold.

Suppose that Ml has a 0 in each row. We make use of the following claims, which hold for all i,j[n]:

  1. for each clause C on P, if t¯i,jC then {ui,u¯i}C;

  2. each xi-resolvent in π contains {ui,u¯i} as a subset;

  3. for each ti,j-resolvent R in π, if xivars(R) then {ui,u¯i}R.

We proceed to show that every row in Ml also has at least one 1. To see this, suppose on the contrary that Ml contains a full 0 row r (this implies that l2, and hence that Ml-1 exists). Note that by definition of resolution there can be at most one element that changes from 1 in Ml-1 to 0 in Ml. Since Ml-1 does not have a 0 in every column, it does not contain a full zero row. Hence it must be the case that the unique element that went from 1 in Ml-1 to 0 in Ml is in row r. Since n2, we deduce that Ml-1 has a 0 in each row, contradicting the minimality of l.

Let i[n]. Since the ith row in Ml contains a 1, there is some j[n] for which t¯i,jCl. From claim (1) it follows that {ui,u¯i}Cl. Moreover, as universal literals accumulate along the path, this means that {ui,u¯i}Cm for each ml. Since the ith row in Ml contains a 0, there exists j[n] such that t¯i,jCl. As t¯i,jC1, there must be a ti,j-resolvent Cl on P with ll. Then we have xivars(Cl) by claim (3). Also, for each ml, Cm is not an xi-resolvent by claim (2). It follows that xivars(Cl). Since i[n] was chosen arbitrarily, we have Xvars(Cl).

Suppose on the other hand that Ml does not contain a 0 in each row. Then Ml contains a 0 in each column. A symmetrical argument, with analogous claims involving the vj,yj variables, then shows that Yvars(Cl).

It remains to prove the three claims.

  1. Observe that each clause in π containing the positive literal ti,j also contains the variable ui (this holds for every axiom and universal literals are never removed). Let C be a clause on the path P for which t¯i,jC, and, for the sake of contradiction, suppose that {ui,u¯i}C. Since ui<Q(n)ti,j, there cannot be ti,j-resolvent on P following C, as such a resolution step is explicitly forbidden in the rules of reductionless LD-Q-Res. This means that t¯i,j occurs in Ck, the final clause of P. This is a contradiction, since Ck is the conclusion of π, which contains no existential literals. Therefore {ui,ui¯}C.

  2. Observe that each clause in π containing xi (resp. x¯i) also contains ui (resp. u¯i) (again, this holds for every axiom and universal literals are never removed). Let R be an xi-resolvent of R1 and R2 in π. Since xiR1 and x¯iR2, we must have uiR1 and u¯iR2. It follows immediately that {ui,u¯i}R.

  3. Observe that each axiom in π containing the positive literal ti,j contains variable xi. Hence, any clause in π that contains literal ti,j but not variable xi must appear after an xi-resolvent on some path, and therefore contains {ui,ui¯} by Claim (2). Now, let R be a ti,j-resolvent of R1 and R2 in π. Suppose that xivars(R), which implies that xivars(R1). Since ti,jR1, we have {ui,u¯i}R1, and it follows that {ui,u¯i}R.

It remains to prove the lower bound formally from the preceding lemmata.

Theorem 28

The squared equality family requires exponential-size reductionless LD-Q-Res refutations.

Proof

Let nN, and let π be a reductionless LD-Q-Res refutation of Inline graphic. We show that |π|2n-1. The size bound is trivially true for n=1, so we assume n2. Put X:={x1,,xn} and Y:={y1,,yn}, and let L:={t¯i,j:i,j[n]} be the long clause from Inline graphic. We call a non-tautological clause S symmetrical iff vars(S)=XY and xiSyiS for each i[n]. (A symmetrical clause represents a total assignment to XY). Note that there are 2n distinct symmetrical clauses.

By Lemma 26, for each symmetrical clause S, there exists a path PS in π in which all existential literals are contained in SL. Moreover, each PS begins at clause L, since every other clause in eq2(n) contains some positive ti,j literal that does not occur in SL. By Lemma 27, on each path P from L in π there exists a clause C for which either Xvars(C) or Yvars(C). It follows that we can define a function f that maps each symmetrical assignment S to a clause f(S) in π for which either proj(S,X)f(S) or proj(S,Y)f(S). Moreover, since distinct symmetrical clauses S1 and S2 satisfy proj(S1,X)proj(S2,X) and proj(S1,Y)proj(S2,Y), each f(S) is the image of at most two distinct symmetrical clauses. Hence, π contains at least 2n-1 clauses.

Close inspection of the lower-bound proof reveals that particular resolution steps are blocked due to the appearance of merged literals in the antecedents (see the proof of claim (1) of Lemma 27). As we noted in Example 18, such steps remain blocked even if both merged literals implicitly represent the same (non-constant) function, in which case the resolution step is actually perfectly sound. As we will see, the M-Res upper-bound construction makes crucial use of the isomorphism of non-constant merge maps.

Short M-Res refutations of Inline graphic

Here we construct short M-Res refutations of the squared equality formulas. The approach is as follows. First, for each i,j[n], obtain a line ({ti,j},Mi,j) by resolving the axioms for the four clauses in eq(n)2 that contain {ti,j}. By the natural application of the merge and select operations, one obtains merge maps Mi,j in which the merge map for ui outputs xi with a single query, the merge map for vj outputs yj with a single query, and all other maps are trivial. Notice that all the non-trivial merge maps for a given universal variable are isomorphic, so these n2 unit clauses can all be resolved against the square clause, utilising the select operation. It is precisely this final step which is unavailable in reductionless LD-Q-Res.

Theorem 29

The squared equality family has O(n2)-size M-Res refutations.

Proof

Let nN. We construct a refutation in two stages. In the first stage we explicitly construct an M-Res derivation π:=L1,,Lk from Inline graphic, where k=2n2. In the second stage, we show that π can be extended to a refutation with a further n2+1 lines.

Stage one. For each h,i,jN we let δ(h,i,j):=(h-1)n2+(i-1)n+j and use L(hij) as an alias for Lδ(h,i,j). Similarly, we let C(hij) be the clause, U(hij) be the merge map for ui, and V(hij) be the merge map for vj appearing on line L(hij). These U(hij) and V(hij) are the only merge maps in π we define explicitly; we consider all others to be defined implicitly as the appropriate trivial merge map.

Letting i,j[n], we define the first 4n2 lines with

graphic file with name 10817_2020_9560_Equ25_HTML.gif

and observe that each of these lines can be introduced as an axiom.

The next 2n2 lines are the result of the natural resolutions over yj. For each i,j[n] we define

graphic file with name 10817_2020_9560_Equ26_HTML.gif
graphic file with name 10817_2020_9560_Equ27_HTML.gif
graphic file with name 10817_2020_9560_Equ28_HTML.gif

Each line L(4, ij) can be derived by resolution from L(0, ij) and L(2, ij); to see this, note that U(0, ij) is clearly isomorphic to U(2, ij) and V(0, ij) is trivially consistent with V(2, ij) (their domains are disjoint), therefore U(4,i,j)=select(U(0,i,j),U(2,i,j)) and

V(4,i,j)=merge(V(0,i,j),V(2,i,j),δ(4,i,j),yj).

A similar argument shows each that L(5, ij) can be derived by resolution from L(1, ij) and L(3, ij).

The final n2 lines are the result of the natural resolutions over xi. For each i,j[n] we define

graphic file with name 10817_2020_9560_Equ29_HTML.gif
graphic file with name 10817_2020_9560_Equ30_HTML.gif

It is easy to see that each L(6, ij) can be derived by resolution from L(4, ij) and L(5, ij), since V(4, ij) is clearly isomorphic to V(5, ij) (an isomorphism is ll+n2) and U(0, ij) is trivially consistent with U(1, ij) (disjoint domains).

Stage two. We now show how π can be extended to a refutation. Let L6:={L(6,i,j):i,j[n]} denote the final n2 lines of π, in each of which appears some unit clause {ti,j}. We observe that, for each a,b,i[n], U(6, ia) is isomorphic to U(6, ib) (an isomorphism is ll+b-a); that is, amongst the lines L6, the non-trivial merge maps for ui are pairwise isomorphic. Similarly, for each j[n], the non-trivial merge maps for vj appearing in L6 are pairwise isomorphic.

Now, a line T, consisting of the clause {t¯i,j:i,j[n]} and a full set of trivial merge maps, can be introduced as an M-Res axiom in a derivation from Inline graphic. From T and L6, in a further n2 steps we obtain a refutation by successively resolving each line in L6 against T, removing a literal t¯i,j each time. All such resolution steps are valid, since the merge map for ui (vj) in any line can be defined as select(Ma,Mb), where Ma and Mb are the merge maps for ui appearing in the antecedent lines. The isomorphism of non-trivial merge maps for ui (vj) is preserved, and ensures that select(Ma,Mb) is defined.

The separation follows immediately from Theorems 28 and 29.

Theorem 30

LD-Q-Res does not p-simulate M-Res on QBF.

Overview of DQBF

In this section, we provide an overview of DQBF, which will help to explain how Merge Resolution is best extended to a DQBF proof system (in Sect. 7).

S-form versus H-form

A DQBF can be written in one of two forms: Skolem-form (S-form) and Herbrand-form (H-form) [2]. To date, most of the DQBF literature has focused on S-form (whether in computational complexity [1, 16], proof complexity [8, 50], and solving [27, 29, 55, 57, 58]), whereas relatively little has been written about H-form [2]. The DQBF solver presented in [25] uses H-form DQBF to facilitate a reduction to QBF. Otherwise, as far as we are aware, existing DQBF solvers use S-form exclusively [52].

We will recall S-form and H-form DQBFs, their semantics, and the transformation operation that relates them.

An S-form dependency quantified Boolean formula (DQBF) is a formula of the form

Φ:=u1umx1(S1)xn(Sn)·ϕ, 1

in which ϕ is a CNF, and each Si is a subset of the universally quantified variables {u1,,um}. S-form DQBF generalises QBF, since the quantifier prefix has a more general specification that allows variable dependencies for the existentials to be written explicitly in the sets Si. QBF is the fragment of S-form DQBF for which the dependency sets are nested subsets, i.e. S1S2Sn.

An S-form DQBF is true if and only if it has a Skolem-function model. A Skolem-function model g for Φ is a set {gi:i[n]} of functions

gi:Si{xi,x¯i}

such that, for each α{u1,,um},

α{gi(αSi):i[n]}satisfiesϕ.

An H-form DQBF is the obvious dual to S-form, namely a formula of the form

Ψ:=x1xnu1(H1)um(Hm)·ϕ,

in which ϕ is a CNF, and each Hi is a subset of the existentially quantified variables {x1,,xn}. Here the Hi express the variable dependencies for the universals, as opposed to the existentials in S-form.

An H-form DQBF is false if and only if it has an Herbrand-function countermodel, which is dual to a Skolem-function model. An Herbrand-function countermodel h for Ψ is a set {hi:i[m]} of functions

hi:Hi{ui,u¯i}

such that, for each β{x1,,xn},

β{hi(βHi):i[m]}falsifiesϕ.

The dual definitions of S-form and H-form DQBF seem perfectly natural, and both sets of formulas generalise QBF in an obvious way. Nonetheless, it was shown in [2] that the situation in terms of semantics is already quite complex. To see this, consider the transformation operation T defined below. (It is a combination of the negation and complement operators defined in [2]. We find it more convenient here to have a single operation.) This operator is a natural map from S-form onto H-form DQBF and from H-form onto S-form DQBF. The T-transform of the S-form DQBF in (1) is the H-form DQBF

T(Φ):=x1xnu1(H1)um(Hm)·ϕ,

where Hi:={xj:uiSj}. Intuitively, in the transformed H-form, a universal variable u depends on the existentials which did not depend on u in the original S-form. The T-transform of the H-form DQBF is defined analogously. (In the notation of [2], for any DQBF Φ, T(Φ)=¬Φ=¬Φ.)

It is easy to see that for any DQBF Φ, T(T(Φ))=Φ.

To see why the T-transform is a natural operation, consider what happens to a QBF. Recall that in an S-form QBF, the dependency sets are nested (S1S2Sn), therefore the dependency sets in the T-transform are also nested (H1H2Hm). In fact, it is not too hard to see that both collections of dependency sets represent the same (linear) QBF prefix. Therefore, the transform of an S-form QBF is just an H-form representation of the same QBF, and this is verified semantically: an S-form QBF has a Skolem-function model (is true) if and only if its transformed H-form does not have an Herbrand-function countermodel (is not false); and it does not have a Skolem-function model if and only if its transform does have an Herbrand-function countermodel. Thus, every QBF Φ is logically equivalent to T(Φ); the only change made by the transformation is from S-form to H-form and vice versa.

But this is not the case in general for DQBF. The authors of [2] partitioned S-form DQBF into four distinct classes:

  • (A)

    those which have a Skolem-function model, but whose transform has no Herbrand-function countermodel.

  • (B)

    those which have no Skolem-function model, but whose transform does have an Herbrand-function countermodel.

  • (C)

    those which have a Skolem-function model, and whose transform also has an Herbrand-function countermodel.

  • (D)

    those which have no Skolem-function model, nor does their transform have an Herbrand-function countermodel.

All QBFs are either type A or B. Type C and D are classes of DQBFs whose semantic properties are markedly different from QBF.

Expansion versus QCDCL

Given what we know about the semantics of DQBF, we pose the following question: What is the impact of the existence of type C and D DQBFs on the transfer of solving techniques from QBF? We argue that the impact is indeed visible in theoretical models of solving. Moreover, it forms a decent explanation for the results that we have seen there.

Figure 6 (reproduced from [13]) depicts what happens when one attempts to lift various QBF calculi to DQBF. All of these systems are refutational calculi for S-form DQBFs; that is, they prove that an S-form DQBF does not have a Skolem-function model.

Fig. 6.

Fig. 6

The simulation order of QBF resolution systems and soundness/completeness of their versions lifted to S-form DQBF

The main message of Fig. 6 (and the conclusion of [13]) is that expansion-based systems lift to S-form DQBF whereas CDCL-based systems do not. Q-Resolution, for example, is too weak (it is not complete for S-form DQBF), whereas long-distance Q-Resolution is too strong (it is not sound).

A reasonable explanation for this goes as follows:

Expansion-based (D)QBF calculi prove the non-existence of Skolem functions, whereas CDCL-based (D)QBF calculi prove the existence of Herbrand functions.

Such an explanation could scarcely be sought in the QBF realm, where the non-existence of a Skolem-function model and the existence of an Herbrand-function countermodel are equivalent. One really needs to consider the behaviour of type C and D formulas to understand that these two things are not equivalent for DQBF.

Whereas our statement is not the kind that can be proved as a theorem, there appears good reason to promote it as a credible hypothesis, since it explains the situation depicted in Fig 6.

Expansion-based systems prove that the universal expansion of a (D)QBF (i.e. a propositional formula) is unsatisfiable. Satisfying assignments for the expansion are in one-one correspondence with Skolem-function models, so a proof of unsatisfiability is a proof of the non-existence of Skolem functions. Thus, the expansion systems Exp+Res and IR-calc should lift quite naturally to refutational systems for S-form DQBFs, whose falsity is witnessed by the non-existence of Skolem functions. And indeed, they lift easily to DQBF, as shown in Fig 6 [13].

Moreover, if CDCL-based systems prove the existence of Herbrand functions, we should expect to see difficulties lifting them to S-form DQBF, because the rules of these systems implicitly work on the T-transformed formulas, which is an H-form DQBF. We know that there exist type C S-form DQBFs that are true, but whose transform also has Herbrand functions, and type D S-form DQBFs that are false, but whose transform does not have Herbrand functions. In the former case we could expect to refute a true formula (unsoundness), in the latter case we find false formulas that we cannot refute (incompleteness). This is precisely what we see in Fig. 6: LD-Q-Res is unsound for S-form DQBF [13], whereas Q-Res is incomplete [2].

Note that IRM-calc, which is considered an expansion-based system, is also unsound for S-form DQBFs. This is because the system is designed to simulate LD-Q-Res, and unfortunately also simulates unsound LD-Q-Res refutations of true S-form DQBFs.

Switching from S-form to H-form

We suggest, then, that it is worthwhile to investigate further the use of H-form DQBF as an input encoding for CDCL-based DQBF solving. At least for theoretical models, this is yet to be investigated. Here we undertake the first such investigation, and we get some positive results: Merge Resolution lifts naturally to a sound and complete CDCL-based refutational proof system on H-form DQBF.

It should be noted that a resolution system for DQBF called Fork Resolution [50] was shown to be sound and complete for S-form DQBF. The system is based on so-called ‘information forks’, and allows the introduction of fresh variables that delegate the responsibility for fork satisfaction between the original variables. Whereas Fork Resolution is clearly a variant of Q-Resolution, it is not clear whether one should call it a CDCL-based system. Certainly, the associated solver DCAQE [55] belongs to the paradigm of clausal abstraction, rather than conflict-driven clause learning. However, we wish to make it clear that switching to H-form is not the only solution to the issues associated with Fig. 6.

Extending merge resolution to H-form DQBF

In this section, we show that M-Res extends naturally to a proof system for H-form DQBF with the addition of a single weakening rule.

For consistency with the QBF definition, we introduce an equivalent notation for H-form DQBF. We write the quantifier prefix of the H-form DQBF

Φ:=x1xnu1(H1)um(Hm)·ϕ

as a triple Q:=(X,U,LQ), where:

  • X={x1,,xn} is the set of existential variables;

  • U={u1,,um} is the set of universal variables;

  • LQ:U(X) is the support set function, which maps each ui to its dependency set Hi.

To lift M-Res to H-form DQBF, we take Φ to be a DQBF in Definition 16 and add an extra case:

  • (c)

    Weakening. There exists an integer a<i such that Ci is an existential superclause of Ca and, for each uU, either (i) Miu=Mau, or (ii) Mau is trivial and Miu:=il for some literal l{u,u¯}.

By ‘existential superclause’ it is meant that vars(Ci)X and CaCi.

Weakening is, in a clear sense, the simplest rule with which one extends M-Res to H-form DQBF. Its function is merely to represent exactly the paths of the countermodel on which the canonical completeness construction is based. In general, the countermodel needs to be represented in full since merge maps must be isomorphic in order to apply the select operation. Note that the DQBF analogue of Proposition 19 is proved easily with an additional case for the weakening rule.

Soundness and completeness

Soundness of M-Res for H-form DQBF is proved in the same way as for QBF, i.e. by showing that the concluding merge maps compute a countermodel.

Lemma 31

Let (,{Mu:uU}) be the conclusion of an M-Res refutation of an H-form DQBF Φ. Then the functions computed by {Mu:uU} form a countermodel for Φ.

Proof

We add an additional case to the inductive step in the proof of Lemma 21. Suppose that Li was derived by weakening. Then there exists an integer a<i such that CaCi and, for each uU, either (i) Miu=Mau, or (ii) Mau is trivial and Miu:=il for some literal l{u,u¯}. Here AiAa, so αAa. For each uU, if u satisfies (i) then liu(α)=lau(α), and if u satisfies (ii) then lau(α)=hi(α). Hence we have ha(α)hi(α). It follows that the restriction of ϕ by αhi(α) contains the empty clause by the inductive hypothesis.

Completeness, on the other hand, cannot be established with an analogue of Theorem 22; DQBF is strictly larger than QBF, and hence simulation of reductionless LD-Q-Res does not guarantee completeness. Our proof rather extends the method by which completeness of reductionless LD-Q-Res was proved in Lemma 5; namely, the construction of a ‘full binary tree’ of resolution steps based on the countermodel, following the prefix order of existential variables.

We give an overview of the construction. Let Φ:=(X,U,LQ)·ϕ be a false DQBF with a countermodel h. For each αX, the assignment αh(α) falsifies some clause Cαϕ by definition of countermodel. Now, consider the M-Res line whose clause is the largest existential clause falsified by α and whose merge maps are constant functions computing h(α). Each such line can be derived in two M-Res steps, by weakening the axiom corresponding to Cα. Moreover, the clauses {Cα:αX} form the leaves of a full binary tree resolution refutation which can be completed using an arbitrary order of the existential pivots X. The merge maps are constructed by merging over the pivot x iff xLQ(u); otherwise the select operation takes the merge map from either antecedent, since the full binary tree structure guarantees that they are isomorphic.

As merge maps essentially represent the structure of resolution steps in the subderivation, it is no surprise that the merge maps in our construction also have a full binary tree structure. This structure is captured by the following definition.

Definition 32

(binary tree merge map) A binary tree merge map for a variable u over a sequence of variables x1,,xn is a function M with domain [2n+1-1] and rule

M(i):=(xlogi+1,2i,2i+1)if1i<2n,liif2ni<2n+1,

where each li{u,u¯}.

At the technical level, we must define existential restrictions for DQBFs and DQBF countermodels. Let Φ:=(X,U,LQ)·ϕ be a DQBF with a countermodel h and let l be a literal with var(l)=xX. The restriction of Φ by l is Φ[l]:=(X\{x},U,LQ)·ϕ[l], where LQ maps each uU to LQ(u)\{x}. The restriction of h by l is h[l]:={hu[l]:uU}, where the functions hu[l]:LQ(u){u,u¯} are defined by hu[l](α):=hu((α{l})LQ(u)).

The construction itself is defined recursively in the completeness proof, combining full binary tree refutations for Φ[x] and Φ[x¯] for some xX with a single resolution step. We use the fact that restrictions preserve countermodels in the following sense.

Proposition 33

Let h be a countermodel for a DQBF Φ:=(X,U,LQ)·ϕ and let l be a literal with var(l)X. Then h[l] is a countermodel for Φ[l].

As the final precursor to the completeness proof, we show that a derivation of the negated literal l¯ and the restricted countermodel h[l] can be obtained easily from a refutation of the restricted DQBF Φ[l]

Proposition 34

Let Φ:=(X,U,LQ)·ϕ be a false DQBF, let l be a literal with var(l)X, and let (,{Mu:uU}) be the conclusion of be an M-Res refutation of Φ[l]. Then there exists an M-Res derivation of ({l¯},{Mu:uU}) from Φ.

Proof

Let π be the refutation with the given conclusion. The desired derivation may be obtained from π simply by adding the literal {l¯} to each clause, applying weakening where necessary, and adjusting the indexing of the merge maps to account for the extra weakening steps.

Lemma 35

Every false H-form DQBF has an M-Res refutation.

Proof

Let Φ:=(X,U,LQ)·ϕ be a false DQBF, and let X:={x1,,xn} where the xi are pairwise distinct. For any M-Res refutation π with conclusion (Ck,{Mku:uU}), let {hu:uU} be the concluding countermodel for π, where the hu are the functions computed by the concluding merge maps Mku. A merge map for uU over LQ(u) is said to be complete if it is isomorphic to a binary tree merge map for u over the sequence

xσ(1),xσ(|LQ(u)|),

which enumerates LQ(u) in increasing index order; that is, σ:[|LQ(u)|][n] is the unique function satisfying {xσ(i):i[|LQ(u)|]}=LQ(u) and i<jσ(i)<σ(j) for each i,j[|LQ(u)|]. By induction on the number n of existential variables, we show that, for each countermodel h for Φ, there exists an M-Res refutation whose concluding countermodel is h and whose concluding merge maps are complete. To that end, let h:={hu:uU} be an arbitrary countermodel for Φ.

For the base case |X|=0, observe that each hu is a constant function with some singleton codomain {lu}. By definition of countermodel, there exists a clause Cϕ such that C={l¯u:uvars(C)}. Applying the axiom rule to C, one obtains a derivation of the line (,{Mu:uU}) in which Mu computes the constant function hu if uvars(C), and is trivial otherwise. With a single weakening step, each trivial Mu can be swapped for a merge map isomorphic to 1lu. Then each Mu is trivially complete and computes the constant function hu.

For the inductive step, let nN. Combining Propositions 33 and 34 with the inductive hypothesis, we deduce that there exist M-Res derivations π and π of the lines ({x¯1},{Mu:uU}) and ({x1},{Mu:uU}) from Φ in which the Mu and Mu are complete merge maps computing hu[x1] and hu[x¯1]. Assume that the lines of π are indexed from 1 to |π| and that those of π are indexed from |π|+1 to |π|+|π|. For each uU, the domains of Mu and Mu are disjoint, so MuMu. If x1LQ(u), then hu[x1]=hu[x¯1], and we must have MuMu since complete merge maps computing the same function must be isomorphic. It follows that the line (,{Mu:uU}) can be derived from Φ, where

Mu:=merge(Mu,Mu,|π|+|π|+1,x1)ifx1LQ(u),Muifx1LQ(u).

It is easy to see that the Mu are complete merge maps computing the hu.

The weakening rule is clearly polynomial-time checkable. Thus the following is immediate from Lemmata 31 and 35.

Theorem 36

M-Res is a proof system for H-form DQBF.

It is natural to consider whether the weakening rule is necessary for completeness. This is indeed the case; there exist false H-form DQBFs that cannot be refuted by M-Res without weakening.

For example, consider the DQBF Φ:=(X,U,LQ)·ϕ in which X:={x1,x2}, U:={u1,u2}, the support set function is given by

LQ(u1)={x1},LQ(u2)={x2},

and the matrix ϕ consists of the clauses

{x¯1,x¯2,u¯1,u¯2},{x1,x2,u1,u2},{x¯1,x2},{x1,x¯2}.

It is easy to see that the only countermodel for Φ sets u1=x1 and u2=x2. Note that the functions computing this unique countermodel have ranges {u¯1,u1} and {u¯2,u2}

Now, let π be a weakening-free M-Res derivation from Φ. We will show that each line in π is of one of three types:

  • A
    The merge maps compute functions with ranges R1A and R2A, where
    {u1}R1A{,u1}and{u2}R2A{,u2};
  • B
    The merge maps compute functions with ranges R1B and R2B, where
    {u¯1}R1B{,u¯1}and{u¯2}R2B{,u¯2};
  • C

    The merge maps compute functions with ranges R1C=R2C={}.

From this it follows that π is not a refutation, because its concluding merge maps do not compute a countermodel.

The axiom line for the clause {x¯1,x¯2,u¯1,u¯2} is type A, the axiom line for the clause {x1,x2,u1,u2} is type B, and the remaining two clauses, which contain no universal literals, are type C. It is easy to see that resolution of a type A line with a type A or C line always yields type A. Similarly, resolution of a type B line with a type B or C line always yields type B. Resolving two type C clauses yields a type C clause. Moreover, type A lines can never be resolved with type B lines; in this case, the merge maps for u1 are non-trivial and non-isomorphic, and similarly for u2, so neither x1 nor x2 is eligible as the pivot variable.

Conclusions and future work

What is new in M-Res?

To the best of our knowledge, M-Res is the first ‘long-distance’ proof system for DQBF. Recent work [13] showed that the DQBF version of LD-Q-Res is not sound, so it is natural to ask how M-Res fares in comparison. We identify three major differences.

Firstly, M-Res works with Herbrand-form DQBFs, whereas the system in [13] was defined for Skolem-form DQBFs (which use support sets for existential variables). Merge maps detail precisely how the Herbrand functions are encoded in the resolution structure of long-distance proofs. One could say that such refutations are ‘proving the existence of Herbrand functions’. For QBF, this is of course equivalent to proving the non-existence of Skolem functions, but that does not carry over to DQBF (in a precise technical sense [2]). From this standpoint, it is natural to refute H-form DQBFs by finding the Herbrand functions that certify the falsity of the formula, and this is exactly what M-Res achieves. On the other hand, [13] takes the approach of refuting S-form DQBFs—which amounts to proving the non-existence of Skolem functions—by looking for Herbrand functions that may exist even if the formula is true.

The second difference is the absence of universal reduction. The difficulty of dealing with universal reduction in the context of DQBF resolution is to some extent addressed in [7], where it is considered in the (closely related [8]) context of dependency schemes. There it is shown that the interplay between universal reduction and merging is problematic, and additional constraints must be placed on universal reduction to prevent unsound inferences. Given that universal reduction is not necessary for completeness, it seems natural to dispense with it entirely.

The third and final difference is the explicit representation of functions in M-Res, versus the function placeholders known as ‘merged literals’ from classical long-distance Q-resolution. Here we argue that the ‘full binary tree’ construction that features in the proofs of Lemmata 5 and 35 is the canonical completeness proof for CDCL-based systems. The explicit representation of functions is key to this construction, since it allows the comparison of non-trivial merge maps. Thus we argue that building strategies into proofs is the natural way to overcome incompleteness.

Relevance to solving

Merge maps may be relevant for QBF and DQBF solving.

In dependency learning for QBF [45], variable dependencies are ignored until clause learning is blocked by an illegal merge. Our work demonstrates that many ‘illegal’ merges are perfectly sound inferences; moreover, M-Res provides a mechanism for identifying such cases based on isomorphism. Thus, it is plausible that incorporating merge maps could increase the scope of dependency learning.

In DQBF, practitioners are still looking for a natural ‘CDCL-based’ (as apposed to ‘expansion-based’) solving paradigm. Our discussion in Sect. 6 suggests one possible reason: namely, the use of Skolem form encodings is not conducive to CDCL-based search. An interesting direction for future work, therefore, would be to experiment with Herbrand-form DQBFs as the standard input format for CDCL-based DQBF solving.

It seems natural, then, to suggest Merge Resolution as the underlying resolution engine in a CDCL-based solver for Herbrand-form DQBF. Conceiving such an implementation would require some work; for example, one would need to store partial strategies with learned clauses, and carry out an efficient isomorphism test. Isomorphism is an easy way to determine the equivalence of two Boolean functions, but in general it seems unlikely that two equivalent functions will have identical representations. This points towards efficient (approximate) equivalence testing as the key to a successful implementation of M-Res.

Complexity of H-form DQBF

Whereas the decision problem for S-form DQBF is known to be NEXP complete [1], the complexity of the decision problem for H-form DQBFs, as far as we are aware, has not been studied. Moreover, the methodology of [1] does not seem appropriate for H-form DQBFs. Since every QBF can be written as an H-form DQBF, the decision problem is certainly PSPACE-hard, and the NEXP upper bound applies for all DQBFs, but its exact complexity remains an interesting open problem.

Acknowledgements

Open Access funding provided by Projekt DEAL. Research was supported by grants from the John Templeton Foundation (Grant No. 60842) and the Carl Zeiss Foundation.

Footnotes

1

There exists associated proof systems for true QBFs [30].

2

Previous DQBF resolution systems either use expansion [13] or extension variables [50].

3

The notion is evident to a greater or lesser degree in all of the papers [4, 7, 23, 44, 46, 54].

4

Reductionless LD-Q-Res p-simulates level-ordered Q-Res by means of a simple construction, and is exponentially separated by the equality formulas [9]. It is also known that reductionless LD-Q-Res and Q-Res are incomparable [47].

O. Beyersdorff: An extended abstract of this article appeared at the proceedings of STACS’19 [10].

Publisher's Note

Springer Nature remains neutral with regard to jurisdictional claims in published maps and institutional affiliations.

References

  • 1.Azhar S, Peterson G, Reif J. Lower bounds for multiplayer non-cooperative games of incomplete information. J. Comput. Math. Appl. 2001;41:957–992. doi: 10.1016/S0898-1221(00)00333-3. [DOI] [Google Scholar]
  • 2.Balabanov V, Chiang H-JK, Jiang J-HR. Henkin quantifiers and Boolean formulae: a certification perspective of DQBF. Theoret. Comput. Sci. 2014;523:86–100. doi: 10.1016/j.tcs.2013.12.020. [DOI] [Google Scholar]
  • 3.Balabanov V, Jiang J-HR. Unified QBF certification and its applications. Form. Methods Syst. Des. 2012;41(1):45–65. doi: 10.1007/s10703-012-0152-6. [DOI] [Google Scholar]
  • 4.Balabanov, V., Jiang, J.-H.R., Janota, M., Widl, M.: Efficient extraction of QBF (counter)models from long-distance resolution proofs. In: Bonet, B., Koenig, S. (eds.) National Conference on Artificial Intelligence (AAAI), pp. 3694–3701. AAAI Press (2015)
  • 5.Benedetti, M.: sKizzo: a suite to evaluate and certify QBFs. In: Nieuwenhuis, R. (ed.) International Conference on Automated Deduction (CADE), Volume 3632 of Lecture Notes in Computer Science, pp. 369–376. Springer (2005)
  • 6.Benedetti M, Mangassarian H. QBF-based formal verification: experience and perspectives. J. Satisf. Boolean Model. Comput. 2008;5(1–4):133–191. [Google Scholar]
  • 7.Beyersdorff, O., Blinkhorn, J. (2016) Dependency schemes in QBF calculi: semantics and soundness. In: Rueher, M. (ed.) International Conference on Principles and Practice of Constraint Programming (CP), Volume 9892 of Lecture Notes in Computer Science, pp. 96–112. Springer
  • 8.Beyersdorff O, Blinkhorn J, Chew L, Schmidt RA, Suda M. Reinterpreting dependency schemes: soundness meets incompleteness in DQBF. J. Autom. Reason. 2019;63(3):597–623. doi: 10.1007/s10817-018-9482-4. [DOI] [PMC free article] [PubMed] [Google Scholar]
  • 9.Beyersdorff, O., Blinkhorn, J., Hinde, L.: Size, cost, and capacity: a semantic technique for hard random QBFs. Log. Methods Comput. Sci. 15(1), 13:1–13:39 (2019)
  • 10.Beyersdorff, O., Blinkhorn, J., Mahajan, M.: Building strategies into QBF proofs. In: Niedermeier, R., Paul, C. (ed.) International Symposium on Theoretical Aspects of Computer Science (STACS), Volume 126 of Leibniz International Proceedings in Informatics (LIPIcs), pp. 14:1–14:18. Schloss Dagstuhl - Leibniz-Zentrum für Informatik (2019)
  • 11.Beyersdorff, O., Bonacina, I., Chew, L.: Lower bounds: from circuits to QBF proof systems. In: Sudan, M. (ed.) ACM Conference on Innovations in Theoretical Computer Science (ITCS), pp. 249–260. ACM (2016)
  • 12.Beyersdorff O, Chew L, Janota M. New resolution-based QBF calculi and their proof complexity. ACM Trans. Comput. Theory. 2019;11(4):26:1–26:42. doi: 10.1145/3352155. [DOI] [Google Scholar]
  • 13.Beyersdorff, O., Chew, L., Schmidt, R.A., Suda, M.: Lifting QBF resolution calculi to DQBF. In: Creignou and Berre [21], pp. 490–499
  • 14.Beyersdorff O, Wintersteiger CM, editors. International Conference on Theory and Practice of Satisfiability Testing (SAT), Volume 10929 of Lecture Notes in Computer Science. Berlin: Springer; 2018. [Google Scholar]
  • 15.Bjørner, N., Janota, M., Klieber, W.: On conflicts and strategies in QBF. In: Fehnker, A., McIver, A., Sutcliffe, G., Voronkov, A. (eds.) International Conference on Logic for Programming, Artificial Intelligence and Reasoning—Short Presentations (LPAR), Volume 35 of EPiC Series in Computing, pp. 28–41. EasyChair (2015)
  • 16.Bubeck, U., Büning, H.K.: Dependency quantified Horn formulas: models and complexity. In: Biere, A., Gomes, C.P. (eds.) International Conference on Theory and Practice of Satisfiability Testing (SAT), Volume 4121 of Lecture Notes in Computer Science, pp. 198–211. Springer (2006)
  • 17.Buss SR. Towards NP-P via proof complexity and search. Ann. Pure Appl. Log. 2012;163(7):906–917. doi: 10.1016/j.apal.2011.09.009. [DOI] [Google Scholar]
  • 18.Cashmore, M., Fox, M., Giunchiglia, E.: Partially grounded planning as quantified Boolean formula. In: Borrajo, D., Kambhampati, S., Oddi, A., Fratini, S. (eds.) International Conference on Automated Planning and Scheduling (ICAPS). AAAI (2013)
  • 19.Cook SA, Nguyen P. Logical Foundations of Proof Complexity. Cambridge: Cambridge University Press; 2010. [Google Scholar]
  • 20.Cook SA, Reckhow RA. The relative efficiency of propositional proof systems. J. Symb. Log. 1979;44(1):36–50. doi: 10.2307/2273702. [DOI] [Google Scholar]
  • 21.Creignou N, Le Berre D, editors. International Conference on Theory and Practice of Satisfiability Testing (SAT). Lecture Notes in Computer Science. Berlin: Springer; 2016. [Google Scholar]
  • 22.Egly U, Kronegger M, Lonsing F, Pfandler A. Conformant planning as a case study of incremental QBF solving. Ann. Math. Artif. Intell. 2017;80(1):21–45. doi: 10.1007/s10472-016-9501-2. [DOI] [Google Scholar]
  • 23.Egly, U., Lonsing, F., Widl, M.: Long-distance resolution: proof generation and strategy extraction in search-based QBF solving. In: McMillan, K.L., Middeldorp, K.L., Voronkov, A. (eds.) International Conference on Logic for Programming, Artificial Intelligence and Reasoning (LPAR), Volume 8312 of Lecture Notes in Computer Science, pp. 291–308. Springer (2013)
  • 24.Faymonville, P., Finkbeiner, B., Rabe, M.N., Tentrup, L.: Encodings of bounded synthesis. In: Legay and Margaria [39], pp. 354–370
  • 25.Finkbeiner, B., Tentrup, L.: Fast DQBF refutation. In: Sinz, C., Egly, U. (eds.) International Conference on Theory and Practice of Satisfiability Testing (SAT), Volume 8561 of Lecture Notes in Computer Science, pp. 243–251. Springer (2014)
  • 26.Fröhlich, A., Kovásznai, G., Biere, A.: A DPLL algorithm for solving DQBF. https://arise.or.at/pubpdf/Algorithm_for_Solving__DQBF_.pdf, presented at Workshop on Pragmatics of SAT (POS) (2012)
  • 27.Fröhlich, A., Kovásznai, G., Biere, A., Veith, H.: iDQ: instantiation-based DQBF solving. In: Le Berre, D. (ed.) Workshop on Pragmatics of SAT (POS), Volume 27 of EPiC Series in Computing, pp. 103–116. EasyChair (2014)
  • 28.Gaspers S, Walsh T, editors. International Conference on Theory and Practice of Satisfiability Testing (SAT). Lecture Notes in Computer Science. Berlin: Springer; 2017. [Google Scholar]
  • 29.Gitina, K., Wimmer, R., Reimer, S., Sauer, M., Scholl, C., Becker, B.: Solving DQBF through quantifier elimination. In: Nebel, W., Atienza, D. (eds.) Design, Automation & Test in Europe Conference (DATE), pp. 1617–1622. ACM (2015)
  • 30.Giunchiglia E, Narizzano M, Tacchella A. Clause/term resolution and learning in the evaluation of quantified Boolean formulas. J. Artif. Intell. Res. 2006;26:371–416. doi: 10.1613/jair.1959. [DOI] [Google Scholar]
  • 31.Heule, M., Seidl, M., Biere, A.: Efficient extraction of Skolem functions from QRAT proofs. In: Conference on Formal Methods in Computer-Aided Design (FMCAD), pp. 107–114. IEEE (2014)
  • 32.Heule MJH, Kullmann O. The science of brute force. Commun. ACM. 2017;60(8):70–79. doi: 10.1145/3107239. [DOI] [Google Scholar]
  • 33.Janota M, Lynce I, editors. International Conference on Theory and Practice of Satisfiability Testing (SAT). Lecture Notes in Computer Science. Berlin: Springer; 2019. [Google Scholar]
  • 34.Janota M, Marques-Silva J. Expansion-based QBF solving versus Q-resolution. Theor. Comput. Sci. 2015;577:25–42. doi: 10.1016/j.tcs.2015.01.048. [DOI] [Google Scholar]
  • 35.Büning HK, Karpinski M, Flögel A. Resolution for quantified Boolean formulas. Inf. Comput. 1995;117(1):12–18. doi: 10.1006/inco.1995.1025. [DOI] [Google Scholar]
  • 36.Klieber, W., Sapra, S., Gao, S., Clarke, E.M.: A non-prenex, non-clausal QBF solver with game-state learning. In: Strichman, O., Szeider, S. (eds.) International Conference on Theory and Practice of Satisfiability Testing (SAT), Volume 6175 of Lecture Notes in Computer Science, pp. 128–142. Springer (2010)
  • 37.Kontchakov, R., Pulina, L., Sattler, U., Schneider, T., Selmer, P., Wolter, F., Zakharyaschev, M.: Minimal module extraction from DL-lite ontologies using QBF solvers. In: Boutilier, C. (ed.) International Joint Conference on Artificial Intelligence (IJCAI), pp. 836–841. AAAI Press (2009)
  • 38.Krajíček J. Bounded Arithmetic, Propositional Logic, and Complexity Theory. Encyclopedia of Mathematics and Its Applications. Cambridge: Cambridge University Press; 1995. [Google Scholar]
  • 39.Legay, Axel, Margaria, Tiziana (eds.): International Conference on Tools and Algorithms for the Construction and Analysis of Systems (TACAS). Lecture Notes in Computer Science, vol. 10205. Springer, (2017)
  • 40.Ling, A.C., Singh, D.P., Brown, S.D.: FPGA logic synthesis using quantified Boolean satisfiability. In: Bacchus, F., Walsh, T. (eds.), International Conference on Theory and Practice of Satisfiability Testing (SAT), Volume 3569 of Lecture Notes in Computer Science, pp. 444–450. Springer (2005)
  • 41.Mangassarian H, Veneris AG, Benedetti M. Robust QBF encodings for sequential circuits with applications to verification, debug, and test. IEEE Trans. Comput. 2010;59(7):981–994. doi: 10.1109/TC.2010.74. [DOI] [Google Scholar]
  • 42.Marques-Silva, J., Malik, S.: Propositional SAT solving. In: Clarke, E.M., Henzinger, T.A., Veith, H., Bloem, R. (eds.) Handbook of Model Checking, pp. 247–275. Springer (2018)
  • 43.Nordström J. On the interplay between proof complexity and SAT solving. SIGLOG News. 2015;2(3):19–44. doi: 10.1145/2815493.2815497. [DOI] [Google Scholar]
  • 44.Peitl, T., Slivovsky, F., Szeider, S.: Long distance Q-resolution with dependency schemes. In: Creignou and Berre [21], pp. 500–518 [DOI] [PMC free article] [PubMed]
  • 45.Peitl, T., Slivovsky, F., Szeider, S.: Dependency learning for QBF. In: Gaspers and Walsh [28], pp. 298–313
  • 46.Peitl, T., Slivovsky, F., Szeider, S.: Polynomial-time validation of QCDCL certificates. In: Beyersdorff and Wintersteiger [14], pp. 253–269
  • 47.Peitl, T., Slivovsky, F., Szeider, S.: Proof complexity of fragments of long-distance Q-resolution. In: Janota and Lynce [33], pp. 319–335
  • 48.QBFEVAL homepage: http://www.qbflib.org/index_eval.php. Accessed 26 Oct 2018
  • 49.Rabe, M.N., Tentrup, L.: CAQE: a certifying QBF solver. In: Kaivola, R., Wahl, T. (eds.) Conference on Formal Methods in Computer-Aided Design (FMCAD), pp. 136–143. IEEE (2015)
  • 50.Rabe, M.N.: A resolution-style proof system for DQBF. In: Gaspers and Walsh [28], pp. 314–325
  • 51.Samulowitz, H., Davies, J., Bacchus, F.: Preprocessing QBF. In: Benhamou, F. (ed.) International Conference on Principles and Practice of Constraint Programming (CP), Volume 4204 of Lecture Notes in Computer Science, pp. 514–529. Springer (2006)
  • 52.Scholl, C., Wimmer, R.: Dependency quantified Boolean formulas: an overview of solution methods and applications—extended abstract. In: Beyersdorff and Wintersteiger [14], pp. 3–16
  • 53.Silva, J.P.M., Lynce, I., Malik, S.: Conflict-driven clause learning SAT solvers. In: Biere, A., Heule, M., van Maaren, H., Walsh, T. (eds.) Handbook of Satisfiability, Volume 185 of Frontiers in Artificial Intelligence and Applications, pp. 131–153. IOS Press (2009)
  • 54.Suda, M., Gleiss, B.: Local soundness for QBF calculi. In: Beyersdorff and Wintersteiger [14], pp. 217–234
  • 55.Tentrup, L., Rabe, M.N.: Clausal abstraction for DQBF. In: Janota and Lynce [33], pp. 388–405
  • 56.Vardi MY. Boolean satisfiability: theory and engineering. Commun. ACM. 2014;57(3):5. doi: 10.1145/2578043. [DOI] [Google Scholar]
  • 57.Wimmer, R., Gitina, K., Nist, J., Scholl, C., Becker, B.: Preprocessing for DQBF. In: Heule, M., Weaver, S. (eds.) International Conference on Theory and Practice of Satisfiability Testing (SAT), Volume 9340 of Lecture Notes in Computer Science, pp. 173–190. Springer (2015)
  • 58.Wimmer, R., Reimer, S., Marin, P., Becker, B.: HQSpre—an effective preprocessor for QBF and DQBF. In: Legay and Margaria [39], pp. 373–390
  • 59.Zhang, L., Malik, S.: Conflict driven learning in a quantified Boolean satisfiability solver. In: International Conference on Computer-Aided Design (ICCAD), pp. 442–449 (2002)

Articles from Journal of Automated Reasoning are provided here courtesy of Springer

RESOURCES