Abstract 1 Introduction 2 Preliminaries 3 Foundations of Separability 4 Unary Case 5 Binary Case 6 Ternary and Beyond 7 Case Study: Graded Modalities 8 Conclusion References

Modal Separation of Fixpoint Formulae

Jean Christoph Jung ORCID TU Dortmund University, Germany Jędrzej Kołodziejski ORCID TU Dortmund University, Germany
Abstract

Modal separability for modal fixpoint formulae is the problem to decide for two given modal fixpoint formulae φ,φ whether there is a modal formula ψ that separates them, in the sense that φψ and ψ¬φ. We study modal separability and its special case modal definability over various classes of models, such as arbitrary models, finite models, trees, and models of bounded outdegree. Our main results are that modal separability is PSpace-complete over words, that is, models of outdegree 1, ExpTime-complete over unrestricted and over binary models, and 2-ExpTime-complete over models of outdegree bounded by some d3. Interestingly, this latter case behaves fundamentally different from the other cases also in that modal logic does not enjoy the Craig interpolation property over this class. Motivated by this we study also the induced interpolant existence problem as a special case of modal separability, and show that it is coNExpTime-complete and thus harder than validity in the logic. Besides deciding separability, we also investigate the problem of efficient construction of separators. Finally, we consider in a case study the extension of modal fixpoint formulae by graded modalities and investigate separability by modal formulae and graded modal formulae.

Keywords and phrases:
Modal Logic, Fixpoint Logic, Separability, Interpolation
Copyright and License:
[Uncaptioned image] © Jean Christoph Jung and Jędrzej Kołodziejski; licensed under Creative Commons License CC-BY 4.0
2012 ACM Subject Classification:
Theory of computation Modal and temporal logics
Editors:
Olaf Beyersdorff, Michał Pilipczuk, Elaine Pimentel, and Nguyễn Kim Thắng

1 Introduction

For given logics ,+, the -separability problem for + is to decide given two +-formulae φ,φ whether there is an -formula ψ that separates φ and φ in the sense that φψ and ψ¬φ. Obviously, a separator can only exist when φ and φ are mutually exclusive, and the problem is only meaningful when is less expressive than +. Intuitively, a separator formulated in a “simpler” logic explains a given inconsistency in a “complicated” logic +. Note that, for logics + closed under negation, -separability generalizes the -definability problem for +: decide whether a given +-formula is equivalent to an -formula. Indeed, φ+ is equivalent to an -formula iff φ and ¬φ are -separable. Since separability is more general than definability, solving it requires an even better understanding of the logics under consideration. Both separability and definability are central problems with many applications in computer science. As seminal work let us only mention definability and separability of regular word languages by first-order logic [26, 29, 9].

In this paper we study definability and separability of formulae of the modal μ-calculus μ𝖬𝖫 [27, 20] by formulae in propositional modal logic 𝖬𝖫. μ𝖬𝖫 is the extension of 𝖬𝖫 with fixpoints that encompasses virtually all specification languages such as 𝖯𝖣𝖫 [12] and 𝖫𝖳𝖫 and 𝖢𝖳𝖫 [3]. Let us consider an example.

Example 1.

Consider the following properties P1,P2,P3 of vertex-labelled trees:

  • P1: there is an infinite path starting in the root on which each point satisfies a;

  • P2: on every path there are only finitely many points satisfying a;

  • P3: on every path at most two points satisfy a.

The properties are expressible in μ𝖬𝖫 but not in 𝖬𝖫, and both P1,P2 and P1,P3 are mutually exclusive. The properties P1,P3 are separated by the 𝖬𝖫-formula ψ=a(aa) which expresses that there is a path starting with three points satisfying a. On the other hand, no 𝖬𝖫-formula separates P1,P2. The intuitive reason for this is that any 𝖬𝖫-formula ψ only sees trees up to depth |ψ|, and one can find two trees with properties P1,P2 which nonetheless look the same up to depth |ψ|. ∎

We explore the definability and separability problems over several classes of models relevant for computer science: all models, words, trees of bounded or unbounded outdegree; as well as restrictions of all these classes to finite models. On top of analyzing the decision problems, we also address the problem of constructing efficient definitions and separators whenever they exist. The starting point for our research is the seminal paper of Otto [24], where he solves modal definability over models of bounded and unbounded outdegree. In this paper, we continue this line of research and establish a fairly complete and interesting picture. Table 1 summarizes our results. We now explain its content further.

Table 1: Overview of our results. All complexity results are completeness results.
all models words binary trees d-ary trees, d3
𝖬𝖫-definability ExpTime [24] PSpace ExpTime [24] ExpTime [24]
𝖬𝖫-separability ExpTime PSpace ExpTime 2-ExpTime
separator construction double exp. single exp. double exp. triple exp.
𝖬𝖫 interpolant existence always always always coNExpTime

The first line essentially repeats Otto’s results; we only add the observation that 𝖬𝖫-definability over words is PSpace-complete. Interestingly, separability is substantially more difficult. The case of words is the easiest one, both in terms of computational complexity and required arguments. Next come the cases of binary and of unrestricted trees. These two classes possess some nice structural properties which (although true for different reasons) enable a common algorithmic treatment. Finally, the cases of trees with outdegree bounded by a number d3 enter the stage. These trees lack the good properties essential for previous constructions which results in higher computational complexity. The hardness result for d3 is interesting for two reasons. First, as it is entirely standard to encode trees of higher outdegree into binary ones, one could expect the ternary (and higher) case to have the same complexity as the binary one. And second, even though there are known cases when separation is provably harder than definability (regularity of visibly pushdown languages is decidable [23, Theorem 19] but regular separability thereof is not [19, Theorem 2.4]), to the best of our knowledge our results are the only such case known in logic.

The complexity landscape for deciding separability is also reflected in the maximal sizes of the separators that we construct. Relying on the well-known connection of μ𝖬𝖫 to automata, we provide effective constructions for the cases of all models, words, and binary trees. It is worth mentioning that equally effective constructions for definability over all models are given in [22], but they do not work for separability. The ternary case follows from a general argument. Our construction of separators over words is optimal. Under mild assumptions (there are at least two modalities) the constructions over binary and over unrestricted trees are optimal as well, but we leave it open whether these assumptions are needed for the lower bounds. In the case of ternary and higher outdegree trees we only conjecture optimality of the constructed separators.

Finally, we observe that 𝖬𝖫 lacks the Craig interpolation property over trees of outdegree bounded by d3. Recall that a Craig interpolant for φφ in some logic is a formula ψ only using the common symbols of φ and φ and such that φψφ. A logic satisfies the Craig interpolation property (CIP) if a Craig interpolant of φφ always exists. It is known that 𝖬𝖫 enjoys CIP over all models and over words [15] and it follows from our techniques that this transfers to binary trees. In contrast and as mentioned above, over ternary and higher-arity trees 𝖬𝖫 lacks the CIP. It is worth mentioning that modal logic over frames of arity bounded by some d has been studied under the name 𝐊altd [4]. Our results imply that 𝐊altd enjoys CIP iff d2. Motivated by the lack of CIP over higher-arity trees, we study the induced interpolant existence problem – determining whether two given 𝖬𝖫-formulae φ,φ admit a Craig interpolant – as a special case of separability. We show it to be coNExpTime-complete over higher arity trees, and thus harder than validity. Interpolant existence has recently been studied for other logics without CIP [18, 1].

As an application of our results for d-ary trees with d3 we additionally present a case study: separability in the graded setting in which we allow counting modalities saying “there are at least k children such that […]” [11]. Counting modalities are a standard extension of modal logic that is especially relevant in applications in knowledge representation for conceptual modeling [2]. We show that 𝖬𝖫-separability of graded μ𝖬𝖫 is 2-ExpTime-complete, while it is ExpTime-complete if we allow counting modalities also in the separator. The intuitive reason for the hardness in the former case is that trees of bounded arity are definable in graded μ𝖬𝖫. This former case is also related with a recent study about separating logics supporting counting quantifiers by logics without these [21].

It is worth to mention that 𝖬𝖫-definability of μ𝖬𝖫-formulae generalizes the boundedness problem which asks whether a formula with a single fixpoint is equivalent to a modal formula. Boundedness has been studied for other logics such as monadic-second order logic [6], datalog [16], and the guarded fragment of first-order logic [5]. Our paper is an extension of the preliminary paper [17].

The paper is organized as follows. After this introduction 1, we set notation and recall basic facts in the preliminary Section 2. Next, we introduce some topic-specific terminology, discuss a relevant construction of Otto, and solve the case of all models in Section 3. In the following Sections 4 and 5 we deal with unary and binary trees, and in Section 6 we solve the most challenging case of trees of outdegree bounded by d3. Section 7 applies our results to the case with graded modalities. The last Section 8 contains conclusions and final remarks.

2 Preliminaries

We recall the main notions about modal logic 𝖬𝖫 and the modal μ-calculus μ𝖬𝖫. For the rest of this paper fix disjoint, countably infinite sets 𝖯𝗋𝗈𝗉 of atomic propositions and 𝖵𝖺𝗋 of variables. The syntax of μ𝖬𝖫 is given by the rule

φ::=τ|¬τ|φφ|φφ|φ|φ|x|μx.φ|νx.φ

where τ𝖯𝗋𝗈𝗉 and x𝖵𝖺𝗋. We assume that formulae of μ𝖬𝖫 are in a normal form such that every x𝖵𝖺𝗋 appears at most once in a formula, and if it does appear then its appearance has a unique superformula ψ beginning with μx or νx. Modal logic 𝖬𝖫 is defined as the fragment of μ𝖬𝖫 with no fixpoint operators μ and ν nor variables. Both in 𝖬𝖫 and μ𝖬𝖫, we use abbreviations like (for a¬a for some a𝖯𝗋𝗈𝗉), nφ (for a formula φ with n leading ’s), and ¬φ. We denote with sig(φ) the set of propositions that occur in φ, and recall that the modal depth of an 𝖬𝖫 formula is the maximal nesting of ,. With 𝖬𝖫n we denote the class of all 𝖬𝖫-formulae of modal depth at most n, and with 𝖬𝖫σn we denote its subclass restricted to signature σ. The size |φ| of a formula φ is the length of φ represented as a string. This choice of the simplest possible measure of size does not matter for most of our results. We will briefly discuss alternative notions of size in the concluding Section 8.

Both 𝖬𝖫 and μ𝖬𝖫 are interpreted in pointed Kripke structures. More formally, a model is a quadruple =(M,vI,,𝗏𝖺𝗅) consisting of a set M called its universe, a distinguished point vIM called the root, an accessibility relation M×M, and a valuation 𝗏𝖺𝗅:M𝒫(𝖯𝗋𝗈𝗉).

The semantics of μ𝖬𝖫 can be defined in multiple equivalent ways. The one most convenient for us is through parity games (see [32] for an introduction). Given a model and a formula φμ𝖬𝖫 we define a semantic game 𝒢(,φ) played between players ve and dam. The positions are M×𝖲𝗎𝖻𝖥𝗈𝗋(φ). The moves depend on the topmost connective. From a position of the shape (v,ψψ) or (v,ψψ) it is allowed to move to either (v,ψ) or (v,ψ). From (v,ψ) and (v,ψ) the allowed moves lead to all (w,ψ) such that vw. In position (v,τ) or (v,¬τ) the game stops and ve wins iff v satisfies the formula component τ or ¬τ, respectively. From (v,μx.ψ) and (v,μx.ψ) the game moves to (v,ψ), and from (v,x) to (v,ψ) where ψ is the unique superformula of x beginning with μx or νx. ve owns positions whose formula component has or as the topmost connective and dam owns all other positions. ve wins an infinite play π if the outermost subformula seen infinitely often in π begins with ν. We say that ,v satisfies φ and write ,vφ if ve wins the game 𝒢(,φ) from position (v,φ). Since is by definition pointed, we abbreviate ,vIφ with φ.

The same symbol denotes entailment: φψ means that every model of φ is a model of ψ. In the case only models from some fixed class 𝐂 are considered we talk about satisfiability and entailment over 𝐂. Let be a subset of μ𝖬𝖫 such as 𝖬𝖫 or 𝖬𝖫σn. If two models and 𝒩 satisfy the same formulae of then we call them -equivalent and write 𝒩.

In the paper we will study models of bounded and unbounded outdegree. The outdegree of a point wM in a model =(M,vI,,𝗏𝖺𝗅) is the number of successors of w in the underlying directed graph G=(M,). We say that has finite outdegree if every point has finite outdegree and bounded outdegree if there is a finite uniform upper bound d on the outdegree of its points. In the latter case, we will call d-ary, and binary or ternary if d=2 or d=3. If d=1, then we call a word. A d-ary model is full if each of its nodes is either a leaf (i.e. has no children) or has precisely d children. A model is a tree if G is a (directed) tree with root vI. We denote with 𝕋d the class of all d-ary tree models. Both 𝖬𝖫 and μ𝖬𝖫 are invariant under bisimulation, and every (d-ary) model is bisimilar to a (d-ary) tree. Hence, we do not loose generality by only looking at tree models.

A prefix of a tree is a subset of its universe closed under taking ancestors. When no confusion arises we identify a prefix NM with the induced subtree 𝒩 of that has N as its universe. The depth of a point is the distance from the root. The prefix of depth n (or just n-prefix) is the set of all points at depth at most n and is denoted by M|n (and the corresponding subtree by |n).

Bisimulations

We define bisimulations and bisimilarity for trees, assuming for convenience that bisimulations only link points at the same depth. Let , be trees and ZM×M a relation between M and M that relates only points of the same depth. Then, Z is a bisimulation between and if it links the roots vIZvI, and for every wZw the following conditions are satisfied:

(𝖺𝗍𝗈𝗆)

𝗏𝖺𝗅(w)=𝗏𝖺𝗅(w),

(𝖿𝗈𝗋𝗍𝗁)

for every vM with wv there is a vM with wv and vZv, and

(𝖻𝖺𝖼𝗄)

for every vM with wv there is a vM with wv and vZv.

A functional bisimulation (also known as bounded morphism) is a function whose graph is a bisimulation. If Z is a functional bisimulation from to then we write Z:𝖻𝗂𝗌 and call a bisimulation quotient of . The bisimilarity quotient of is a quotient of such that if Z:′′ then =′′. It follows from analogous results for arbitrary models that every tree 𝕋d has a unique (up to isomorphism) bisimilarity quotient 𝕋d and that two trees are bisimilar iff their bisimilarity quotients are isomorphic.

Further, for every n and every subset σ𝖯𝗋𝗈𝗉 of the signature we consider a restricted variant of bisimulations called (σ,n)-bisimulations. In a (σ,n)-bisimulation the 𝖺𝗍𝗈𝗆 condition is only checked with respect to σ and the 𝖻𝖺𝖼𝗄 and 𝖿𝗈𝗋𝗍𝗁 conditions only for points at depth smaller than n. Formally, a relation ZM×M is a (σ,n)-bisimulation if it is a bisimulation between the n-prefixes of the σ-reducts of ,. We call a (σ,n)-bisimulation between , a (σ,n)-isomorphism if it is bijective on the n-prefixes of ,. We write σn if there exists a (σ,n)-bisimulation between and and σn if there is a (σ,n)-isomorphism between them. Crucially, over every class 𝐂 of models and for every finite σ the equivalences 𝖬𝖫σn and σn coincide, for every n.

Automata

We exploit the well-known connection of μ𝖬𝖫 and automata that read tree models. A nondeterministic parity tree automaton (NPTA) is a tuple 𝒜=(Q,Σ,qI,δ,𝗋𝖺𝗇𝗄) where Q is a finite set of states, qIQ is the initial state, Σ=𝒫(σ) for some finite set σ𝖯𝗋𝗈𝗉, 𝗋𝖺𝗇𝗄 assigns each state a priority, and δ is a transition function of type:

δ:Q×Σ𝒫(Qd),

where Qd denotes the set of all tuples over Q of length at most d. A run of 𝒜 on a tree is an assignment ρ:MQ sending the root of the tree to qI and consistent with δ in the sense that (ρ(v1),,ρ(vk))δ(ρ(v),𝗏𝖺𝗅(v)σ) for every point v with children v1,,vk. On occasion when considering trees of unbounded outdegree we will use automata with transition function of type δ:Q×Σ𝒫(𝒫(Q)). Then, consistency of ρ with δ means that {ρ(v)|vV}δ(ρ(v),𝗏𝖺𝗅(v)σ) for every v with a set V of children. In either case, we call the run ρ accepting if for every infinite path v0,v1 in the sequence 𝗋𝖺𝗇𝗄(ρ(v0)),𝗋𝖺𝗇𝗄(ρ(v1)), satisfies the parity condition. We write 𝒜 in case 𝒜 has an accepting run on . An automaton that is identical to 𝒜 except that the original initial state is replaced with q is denoted 𝒜[qIq]. The size of an automaton 𝒜 is the number of its states and is denoted by |𝒜|.

An NPTA 𝒜 is equivalent to a formula φμ𝖬𝖫 over a class 𝐂 of trees when φ iff 𝒜 for every tree 𝐂. We rely on the following classical result (see for example the discussion in [31] and the well-presented Dealternation Theorem 5.7 in [7]):

Theorem 2.

For every μ𝖬𝖫-formula φ and class 𝐂 of trees, we can construct an NPTA with exponentially many states equivalent to φ over 𝐂. The construction takes exponential time when 𝐂𝕋d for some d, and doubly exponential time in the unrestricted case.

3 Foundations of Separability

We start with recalling the notion of separability and discuss some of its basic properties.

Definition 3.

Assume a subset of all μ𝖬𝖫 formulae. Given φ,φμ𝖬𝖫, an -separator of φ,φ is a formula ψ with φψ and ψ¬φ. If additionally sig(ψ)σ for some signature σ, ψ is called an σ-separator.

The -separability problem is to determine, given formulae φ,φμ𝖬𝖫 and a signature σ, if they admit an σ-separator ψ. -definability is the special case of -separability in which φ=¬φ, since an -separator of φ,¬φ is equivalent to φ. All notions can be relativized to a class 𝐂 of models by considering entailment over that class. We investigate 𝖬𝖫-separability and 𝖬𝖫-definability over different classes of models. The reader may have expected the problems to be defined without restrictions on σ, but in fact such versions of the problems are special instances of our problems with σ=sig(φ)sig(φ). Conversely, all lower bounds already hold for such special instances.

We start with observing that, by the tree model property and the finite model property of μ𝖬𝖫, ψ is an 𝖬𝖫σ-separator of φ,φ (over all models) iff ψ is an 𝖬𝖫σ-separator of φ,φ over trees iff ψ is an 𝖬𝖫σ-separator of φ,φ over finite models. Thus, separability coincides over all these classes. Moreover, with the help of the μ𝖬𝖫-formula θ=νx.x expressing the existence of an infinite path originating in the root, 𝖬𝖫-separability over finite trees reduces to 𝖬𝖫-separability over all models. More formally:

Lemma 4.

Let φ,φμ𝖬𝖫 and ψ𝖬𝖫. Then ψ is an 𝖬𝖫σ-separator of φ,φ over finite trees iff ψ is an 𝖬𝖫σ-separator of φ¬θ,φ¬θ. This is also true inside 𝕋d, for d.

This lemma allows us to transfer all upper bounds obtained in the paper also to the restrictions of the classes to finite models. The lower bounds do not follow from this lemma, but analyzing the proofs yields that they actually work as well. Thus, in the rest of the paper we focus on the classes of all models and 𝕋d, for d.

The starting point for the technical developments in the paper are model-theoretic characterizations for separability. Similar to what has been done in the context of interpolation, see for example [28], they are given in terms of joint consistency, which we introduce next. Let R be a binary relation on some class of models, such as (σ,n)-isomorphism σn or 𝖬𝖫σn-equivalence 𝖬𝖫σn. We call two formulae φ,φ joint consistent up to R (in short joint R-consistent) if there are models φ and φ with R(,). For technical reasons we will sometimes also talk about joint consistency of automata 𝒜,𝒜 in place of formulae φ,φ. Joint R-consistency over a class 𝐂 of models is defined by only looking at models from 𝐂. Clearly, if RR and 𝐂𝐂 then joint R-consistency over 𝐂 implies joint R-consistency over 𝐂. We use the following standard equivalence:

φ,φ are not 𝖬𝖫σn-separable over 𝐂 φ,φ are joint σn-consistent over 𝐂. (𝖡𝖺𝗌𝖾)

for every φ,φμ𝖬𝖫, n, finite σ, and class 𝐂. The implication from right to left is immediate. The opposite one follows from the observation that for every n and finite σ there are only finitely many equivalence classes of σn, and each such class is fully described with a single modal formula.

Let us illustrate how Equivalence (𝖡𝖺𝗌𝖾) is used to solve 𝖬𝖫-separability. Let φ1 and φ2 be μ𝖬𝖫-formulae expressing the respective properties P1 and P2 from Example 1. Let be an infinite path in which every point satisfies a, and let n be a finite path of length n in which every point satisfies a. Then, for each n the models ,n witness joint n-consistency of φ1,φ2. By Equivalence (𝖡𝖺𝗌𝖾) this means that φ1,φ2 are not 𝖬𝖫n-separable for any n, and thus not 𝖬𝖫-separable at all.

Definability is a special case of separability. Since the tools used for solving definability are a starting point for our work, we recall them now.

Modal Definability: A Recap

In his seminal paper [24] Otto showed that 𝖬𝖫-definability of μ𝖬𝖫-formulae is ExpTime-complete over all models and over 𝕋d for every d2.

Theorem 5 ([24, Main Theorem and Proposition 5]).

Over the class of all models, as well as over 𝕋d for every d2, 𝖬𝖫-definability of μ𝖬𝖫-formulae is ExpTime-complete.

We start by recalling and rephrasing Otto’s construction and fixing a small mistake in the original proof. The lower bound follows by an immediate reduction from satisfiability of μ𝖬𝖫-formulae. We look at the upper bound. The first step is the following lemma, which is the heart of [24, Lemma 2].

Lemma 6.

For every φμ𝖬𝖫 and n,d the following are equivalent:

  1. 1.

    φ,¬φ are joint σn-consistent over 𝕋d.

  2. 2.

    φ,¬φ are joint σn-consistent over 𝕋d.

The lemma is true, but its proof in [24] is mistaken. The problem there is that the construction duplicates subtrees and hence may turn d-ary models into ones with outdegree greater than d. We present an easy alternative proof.

Proof.

Only the implication 1  2 is nontrivial. To prove it assume d-ary φ, 𝒩¬φ with σn𝒩 and assume towards contradiction that φ,¬φ are not σn-consistent over 𝕋d. We have σn|nσ where σ is the σ-reduct of , and 𝕋d is the bisimilarity quotient of its n-prefix |nσ. By the assumption that φ,¬φ are not joint σn-consistent, φ implies |nσφ. By invariance of φ under , this in turn implies φ. We construct 𝒩¬φ symmetrically. By definition, σn𝒩 means that |nσ and 𝒩|nσ are bisimilar, which is equivalent to saying that their bisimilarity quotients and 𝒩 are isomorphic, and hence (σ,n)-isomorphic. Thus, ,𝒩 witness joint σn-consistency of φ,¬φ over 𝕋d, a contradiction.

Using automata-based techniques we to decide if Item 2 in Lemma 6 holds for all n.

Proposition 7.

For every parity automata 𝒜,𝒜 and d: 𝒜,𝒜 are joint σn-consistent over 𝕋d for all n iff 𝒜,𝒜 are joint σm-consistent over 𝕋d for m=|𝒜|+|𝒜|+1. The latter condition can be checked in time polynomial in |𝒜|+|𝒜|.

Proof (Sketch).

Due to well-known relativization techniques we do not loose generality by only running 𝒜,𝒜 on full d-ary trees with no leaves. Let L be a language of finite full d-ary trees over σ such that L iff is a prefix of a reduct of a model of 𝒜. Let L be an analogous language for 𝒜. The tallness of a finite tree is the minimal distance from the root to a leaf. Observe that 𝒜,𝒜 are σn-consistent over 𝕋d iff LL contains a tree of tallness n. Thus, it suffices to check if LL contains trees of arbitrarily high tallness. To that end construct an automaton recognizing LL of size polynomial in |𝒜|+|𝒜|. An easy pumping argument shows that the language LL of contains trees of arbitrarily high tallness iff it contains a tree of tallness m=||+1. To test the latter condition it is enough to inductively compute a sequence S1S2S||+1 of subsets of states of , where Si is the set of all states q such that [qIq] recognizes a tree of tallness at least i.

We are ready to solve 𝖬𝖫-definability over 𝕋d in exponential time. Assume μ𝖬𝖫-formula φ. For every n, we know by Equivalence (𝖡𝖺𝗌𝖾) that φ is equivalent over 𝕋d to some ψ𝖬𝖫σn iff φ,¬φ are not joint σn-consistent over 𝕋d. By Lemma 6 this is equivalent to the lack of joint σn-consistency of φ,¬φ over 𝕋d. By Theorem 2 we can compute exponentially-sized automata 𝒜, 𝒜 equivalent to φ and ¬φ over 𝕋d. It follows that φ is not 𝖬𝖫σ-definable over 𝕋d iff 𝒜,𝒜 are joint σn-consistent over 𝕋d for every n. The last condition is decided using Proposition 7. The runtime of our algorithm is polynomial in |𝒜|+|𝒜|, and thus exponential in |φ|. This proves the part of Theorem 5 about 𝕋d. The remaining part concerning unrestricted models is a special case of Theorem 9, which we will prove next.

Modal Separation: the Unrestricted Case

Over unrestricted models, separability turns out to be only slightly more complicated than definability. Lemma 6 becomes false if ¬φ is replaced with arbitrary φ (which would be the statement relevant for separability). We have the following lemma, however.

Lemma 8.

For every φ,φμ𝖬𝖫 and n the following are equivalent:

  1. 1.

    φ,φ are joint σn-consistent over all models.

  2. 2.

    φ,φ are joint σn-consistent over 𝕋d, where d=|φ|+|φ|.

Proof.

The implication (1)(2) is immediate. To prove the other one (1)(2) consider an intermediate property:

φ,φ are joint σn-consistent over all models. (1.5)

The implication (1)(1.5) can be read off from Otto’s original proof. The remaining one (1.5)(2) is a special case of a stronger claim which we prove later: the implication (3)(4) of Lemma 27. Lemma 8 allows us to solve 𝖬𝖫-separability in exponential time.

Theorem 9.

Over all models, 𝖬𝖫-separability of μ𝖬𝖫-formulae is ExpTime-complete.

Proof.

The proof is almost the same as our proof of Theorem 5. The only difference is that we consider an arbitrary φ in place of ¬φ, and hence use Lemma 8 in place of Lemma 6. Apart from deciding separability we also construct separators when they exists. Given a subset of μ𝖬𝖫 formulae, φμ𝖬𝖫, and ψ, we call ψ an -uniform consequence of φ if ψθ for every θ such that φθ. The notion relativizes to a fixed class 𝐂 of models by only considering entailment over that class. Observe that if φ,φ are -separable and ψ is an -uniform consequence of φ then ψ is an -separator for φ,φ. The same is true over any class 𝐂.

Note that it follows from the proof of Theorem 9 that if φ,φ are 𝖬𝖫-separable then they admit a separator of modal depth n at most exponential in |φ|+|φ|. It follows that constructing an 𝖬𝖫σ-separator for φ,φ boils down to constructing an 𝖬𝖫σn-uniform consequence of φ. A naive construction which always works is to take the disjunction of all 𝖬𝖫σn-types consistent with φ over 𝐂. Here, by an 𝖬𝖫σn-type we mean a maximal consistent subset of 𝖬𝖫σn. Since up to equivalence there are only finitely many formulae in 𝖬𝖫σn, each 𝖬𝖫σn-type can be represented as a single 𝖬𝖫σn-formula and the mentioned disjunction ψ is well-defined. This construction is non-elementary in n over all models and doubly exponential in n over models of bounded outdegree.

We present an efficient construction of 𝖬𝖫σn-uniform consequences. The construction works over unrestricted models, over 𝕋1 and over 𝕋2 but not over 𝕋d for d3. Since in the following Section 4 we will provide a more efficient construction for 𝕋1, now we only look at the unrestricted and binary case. For convenience, we construct 𝖬𝖫σn-uniform consequences of automata instead of formulae, with definition adapted in an obvious way.

Proposition 10.

Let 𝐂 be the class of all models or 𝕋2. Assume an NPTA 𝒜 over 𝐂, a signature σ and n. An 𝖬𝖫σn-uniform consequence of 𝒜 over 𝐂 can be constructed in time |A|O(n|𝒜|) if 𝐂 is the class of all models and in time 2O(n|A|) if 𝐂=𝕋2.

Proof.

Let 𝒜 be an NPTA. Let =(Q,Σ,qI,δ,𝗋𝖺𝗇𝗄) be an automaton of the same size recognizing σ-reducts of models of 𝒜. A formula ψ is an 𝖬𝖫σn-uniform consequence of 𝒜 over 𝐂 iff it is an 𝖬𝖫n-uniform consequence of over 𝐂. Thus, it suffices to construct the latter.

We construct ψn,q for every qQ and n by induction on n. For the base case we put:

ψ0,q={cΣ|there is 𝒩𝐂 with 𝒩[qIq] and 𝒩c}

For the induction step define:

ψn+1,q=cΣSδ(q,c)c{ψn,p|pS}

where Φ is an abbreviation for θΦθθΦθ. Assume 𝐂 is either the class of all models or 𝕋2. The construction preserves the following invariant:

ψn,q  there exists 𝒩𝐂 with 𝒩[qIq] and n𝒩 (1)

for every structure 𝐂. Hence, ψn,qI is an 𝖬𝖫σn-uniform consequence of 𝒜 over 𝐂. It is routine to check that in either case the formula has the right size.

The proof of (1) proceeds by an easy induction, with slightly different details for the cases of binary and of unrestricted models. It is worth to point out, however, that the implication from left to right would not be valid over 𝕋d with d3.

Given the exponential construction of automata from Theorem 2 and the exponential upper bound on modal depth n of separators, Proposition 10 yields an efficient construction of separators.

Theorem 11.

If φ,φ are 𝖬𝖫σ-separable, then one can compute an 𝖬𝖫σ-separator in time doubly exponential in |φ|+|φ|.

It is not difficult to show that, in the presence of at least two accessibility relations 1,2, the construction is optimal: one can express in μ𝖬𝖫 that the model embeds a full binary tree of depth 2n and in which each inner node has both a 1- and a 2-successor. Using standard techniques, one can show that any modal formula expressing this property is of doubly exponential size [13]. Whether having two accessibility relations is necessary for this lower bound is an interesting question which we leave open.

It is interesting to note that the separators we compute are not the logically strongest separators and, in fact, strongest separators do not even have to exist.

Example 12.

Consider φ=θ from before and φ= For every n, the modal formula n separates φ from φ, and mn whenever mn.

The remaining open cases are the problems of 𝖬𝖫-separability (and separator construction) over 𝕋d for d1. We investigate the cases of unary (d=1), binary (d=2), and higher maximal outdegree (d3) in turn. We emphasize that the outdegree d is not a part of the input but rather a property of the considered class of models.

4 Unary Case

We first investigate 𝖬𝖫-separability over 𝕋1, that is, models that are essentially words. Note that satisfiability of μ𝖬𝖫 over words is PSpace-complete (an upper bound follows, e.g., via the translation to automata and the lower bound is inherited from 𝖫𝖳𝖫 [30, Theorem 4.1]) which suggests that also definability and separability could be easier. Indeed, we show:

Theorem 13.

𝖬𝖫-definability and 𝖬𝖫-separability of μ𝖬𝖫-formulae is PSpace-complete over 𝕋1.

Proof.

The lower bound is by a reduction from satisfiability, and applies to definability.

Given formulae φ,φμ𝖬𝖫 and a subset of the signature σ, consider the set of finite words L={W𝒫(σ)| W is a σ-reduct of a prefix V of some model U of φ}. Let L be a similar language defined for φ. Two unary models are bisimilar iff they are identical. Hence, by Equivalence (𝖡𝖺𝗌𝖾) the formulae φ,φμ𝖬𝖫 are not 𝖬𝖫σ-separable over 𝕋1 iff LL is infinite. It is standard to define a finite automaton 𝒜 recognizing LL and check if its language is infinite (which is equivalent to checking if LL contains input longer than |𝒜|). To do it in polynomial space, we nondeterministically guess the long input, letter by letter, and only remember the current state and a binary counter measuring the length of the input guessed so far.

We conclude this section with proving that 𝖬𝖫σ-separators can be constructed in exponential time and are thus of at most exponential size. Note that this is optimal, since over 𝕋1, μ𝖬𝖫 is exponentially more succinct than 𝖬𝖫. Indeed, it is standard to implement an exponential counter using a polynomially sized μ𝖬𝖫-formula.

Theorem 14.

If φ,φμ𝖬𝖫 are 𝖬𝖫σ-separable over 𝕋1, then one can compute an 𝖬𝖫σ-separator in time exponential in |φ|+|φ|.

As argued in the previous section, it suffices to construct an 𝖬𝖫n-uniform consequence of the NPTA equivalent to φ, which we do next.

Proposition 15.

Let 𝒜 be an NPTA over 𝕋1 with states, n, and σ a signature. An 𝖬𝖫σn-uniform consequence of 𝒜 over 𝕋1 can be constructed in time polynomial in n, σ, and .

Proof.

As argued in the previous section, it suffices to construct an 𝖬𝖫n-uniform consequence of the NPTA  which recognizes precisely the σ-reducts of models of 𝒜. Let have states Q. By construction of , we have |Q|=. As an auxiliary step, we define for every p,qQ and mn a formula ψp,qm𝖬𝖫σn such that for every 𝕋1:

ψp,qmthere is a run of  from p to q over the m-prefix of . (2)

The ψpqm are defined inductively with the base cases (m1) read off from , and using divide and conquer in the inductive step (m>1), to keep the formulae small. More formally, we define ψpqm for m>1 and all p,qQ by taking:

ψpqm =qQ(ψpqm/2m/2ψqqm/2)

It is routine to verify that ψpqm satisfies (2) and is of size |ψpqm|O(|Q|m2). Based on the ψpqm, one can define a formula ψn that describes all possible prefixes of length n of models of , and thus is the sought 𝖬𝖫σ-uniform consequence of . One can think of ψn as the disjunction of formulae ψq0qn for q0 the initial state of , but the full construction is slightly more involved since models accepted by might be also shorter than n.

5 Binary Case

We next handle the binary case 𝕋2. The key observation here is that, between full binary trees, bisimilarity entails isomorphism.

Proposition 16.

Assume full binary trees ,𝕋2. If and are σ-bisimilar then they are σ-isomorphic.

Proof.

By definition a σ-bisimulation between two models is a bisimulation between their reducts to σ, and σ-isomorphism is such a bisimulation which is additionally bijective. It therefore suffices to show that if , are full binary trees and Z is a bisimulation between them then there is a bijective bisimulation ZZ. We pick such Z inductively starting with the pair of roots (vI,vI). The key observation is that if v has children v1,v2 and w has children w1,w2 and vZw then either (i) v1Zw1 and v2Zw2 or (ii) v1Zw2 and v2Zw1 (the cases are not exclusive). Proposition 16 can be used to prove the Craig interpolation property of 𝖬𝖫 over 𝕋2 and implies the following separability-variant of Lemma 6 over 𝕋2.

Lemma 17.

For every φ,φμ𝖬𝖫 and n the following are equivalent:

  1. 1.

    φ,φ are joint σn-consistent over 𝕋2.

  2. 2.

    φ,φ are joint σn-consistent over 𝕋2.

Proof.

We show only the nontrivial implication 1  2. Assume binary φ, φ with σn. Let 𝒩φ and 𝒩φ be full binary trees obtained from and by duplicating subtrees. By Proposition 16, 𝒩σn𝒩 which proves 2. Similarly to the definability case, Lemma 17 combined with Equivalence (𝖡𝖺𝗌𝖾) and Proposition 7 immediately give an exponential procedure for separability. Since the lower bound is inherited from definability, we get the following result.

Theorem 18.

𝖬𝖫-separability and 𝖬𝖫-definability of μ𝖬𝖫-formulae is ExpTime-complete over 𝕋2.

With the same argument as for Theorem 11 we use Proposition 10 to conclude:

Theorem 19.

If φ,φ are 𝖬𝖫σ-separable over 𝕋2, then one can compute an 𝖬𝖫σ-separator in time doubly exponential in |φ|+|φ|.

6 Ternary and Beyond

In this section we address the case of models with outdegree bounded by a number d3. We illustrate that this case behaves differently as it lacks the Craig interpolation property.

Example 20.

Consider 𝖬𝖫-formulae φ=(ab)(a¬b) and φ=(¬ac)(¬a¬c). Clearly, φ¬φ over 𝕋3. Observe that models , in Figure 1 witness that φ,φ are joint {a}-consistent and thus joint {a}n-consistent for every n. By Equivalence (𝖡𝖺𝗌𝖾) there is no 𝖬𝖫{a}-separator, which is nothing else than a Craig interpolant. ∎

Figure 1: Witness of joint consistency: dashed lines and colors indicate the {a}-bisimulation.

Motivated by the lack of the Craig interpolation property, we study the 𝖬𝖫-interpolant existence problem: given φ,φ𝖬𝖫 and signature σ, decide whether there is an 𝖬𝖫σ-separator of φ,¬φ, that is, ψ𝖬𝖫σ with φψφ. Craig 𝖬𝖫-interpolant existence is the special case in which σ=sig(φ)sig(φ). Observe that 𝖬𝖫-interpolant existence is the special case of 𝖬𝖫-separability of μ𝖬𝖫-formulae in which the input to the separability is restricted to 𝖬𝖫-formulae. We show that already 𝖬𝖫-interpolant existence over 𝕋3 is harder than 𝖬𝖫-separability of μ𝖬𝖫-formulae over arbitrary models.

Theorem 21.

For d3, 𝖬𝖫-interpolant existence over 𝕋d is coNExpTime-complete. Hardness already applies to Craig 𝖬𝖫-interpolant existence over 𝕋d.

Proof.

The upper bound is easy to establish based on the observation that φ,¬φ of modal depth at most m do not admit an 𝖬𝖫σ-separator over 𝕋d iff they are joint σm-consistent over 𝕋d. The witness , of joint σm-consistency of φ,¬φ can assumed to be of depth m. Such models are of exponential size (they have at most dm points) and can thus be guessed by a non-deterministic exponential time bounded Turing machine.

The lower bound is more intriguing and relies on an extension of Example 20. Reconsidering the example it is important to note that in every witness , of joint {a}n-consistency of φ,φ, there are two successors of vI that are bisimilar to the same successor of vI. We extend the idea and enforce exponentially many bisimilar points. More precisely, consider families (ψi)i, (ψi)i of modal formulae inductively defined as follows:

ψ0 =ψ0=
ψi+1 =(abi)(a¬bi)(a(ψi(bij<ijbi)(¬bij<ij¬bi)))
ψi+1 =(¬ac)(¬a¬c)(aψi)

Clearly, the size of ψi,ψi is polynomial in i. Moreover, by induction on i, it is readily verified that for every i, for every ,𝕋3 with ψi, ψi, and every ({a},i)-bisimulation S witnessing {a}i, there are points w0,,w2i1 in depth i in and a point w^ in depth i in such that (wj,w^)S for all j and such that distinct wj,wk can be distinguished by some proposition in b0,,bi1. Intuitively, this means that ψi,ψi enforce in joint {a}i-consistent models , that contains 2i points w0,,w2i1 which are all linked to the same point w^ in . We exploit this link to synchronize information between the wj, following a strategy that has recently been used to show coNExpTime-hardness for interpolant existence in some description logics [1].

We reduce a NExpTime-complete tiling problem [14]: Given a set Δ of tile types and horizontal and vertical compatibility relations H,VΔ×Δ, and some n in unary, decide whether one can tile the 2n×2n torus with tiles from Δ complying with H,V. Given Δ,H,V,n, we define formulae φn=ψ2n2nχn, φn=ψ2n2nχn of modal depth m and with common signature σ=sig(φn)sig(φn) such that

Δ,H,V,n has a solution  φn,φn are joint σm-consistent.

To explain the idea, let , witness joint σm-consistency of φn,φn. The gadget formulae ψ2n,ψ2n enforce 22n points w0,,w22n1 in depth 2n in which are all linked via the bisimulation to a single point w^ in . These 22n points shall represent the 2n×2n cells of the torus. The intended solution of the tiling problem is represented via propositions pdσ, for each dΔ. To synchronize them we proceed as follows. Using the 2n propositions b0,,b2n1 (which are not in σ), we can associate coordinates (xi,yi){0,,2n1}×{0,,2n1} to each point wi in the torus. To understand the purpose of χn,χn, suppose for a moment that the outdegree of the points w^ and the wi is at most 22n (instead of 3). Then we could proceed by enforcing (via χn) below each wi with coordinates (xi,yi) three successors vi1,vi2,vi3 such that

  • vi1, vi2, vi3 have coordinates (xi,yi), (xi,yi+1), and (xi+1,yi), respectively;

  • the coordinates of the vij are made visible using propositions in σ;

  • vi1,vi2,vi3 satisfy pd1,pd2,pd3 for d1,d2,d3Δ such that (d1,d2)V and (d1,d3)H.

These three successors stipulate bisimilar successors of w^. Since each point in the torus is stipulated three times as successor of some wi and since the outdegree of w^ is restricted to 22n, the three copies of the same point satisfy the same proposition pd. By the last item above, the selected propositions comply with V,H and thus represent a solution to the tiling problem. Now, since the outdegree below w^ is at most 3 (and not 22n as assumed), the χn,χn have to be a bit more complicated, but the idea remains the same.

We show next that the situation for the full separability problem is even worse.

Theorem 22.

For every d3, 𝖬𝖫-separability of μ𝖬𝖫-formulae over 𝕋d is 2-ExpTime-complete.

Thus, over 𝕋d for d3, 𝖬𝖫-separability is provably harder than 𝖬𝖫-definability, c.f. Theorem 5. Both the upper and the lower bound of Theorem 22 are non-trivial; we provide proof sketches in the following two subsections. Before doing that let us conclude this part with separator construction.

Theorem 23.

If φ,φ are 𝖬𝖫σ-separable over 𝕋d, d3, then one can compute an 𝖬𝖫σ-separator in time triply exponential in |φ|+|φ|.

Proof.

(Sketch) It follows from the upper bound proof of Theorem 22 that, if φ,φ admit an 𝖬𝖫σ-separator, then they admit one of modal depth bounded doubly exponentially in |φ|+|φ|. Observe that over the signature of φ and φ there are only triple exponentially many trees of fixed outdegree d and double exponential depth, and that each such tree is characterized by a modal formula of triply exponential size. The sought separator is then the disjunction of all such formulae consistent with φ.

6.1 Lower Bound for Theorem 22

We reduce the word problem of exponentially space bounded alternating Turing machines (ATMs), which is known to be 2-ExpTime-complete [8]. Informally, the states of such ATMs are partitioned into universal states Q and existential states Q. Configurations of ATMs are defined as usual, but computations are not sequences of configurations but trees of configurations such that an existential configuration has exactly one successor labeled with a universal configuration and a universal configuration has exactly two successors labeled with existential configurations. A computation tree for an input w is a tree whose root is labeled with the initial configuration and such that successor nodes contain successor configurations. w is accepted if there is a computation tree in which each path is infinite (this acceptance condition is slightly non-standard, but eases the proof).

The reduction relies on the same gadget formulae (ψi)i,(ψi)i as used in the proof of Theorem 21 and additionally uses ideas for showing 2-ExpTime-hardness for recently studied interpolant existence problems for description logics [1]. For a given ATM 𝔄 and input w of length n, we construct formulae φn=ψnnχ,φn=ψnχ such that

φn,φn are joint σm-consistent for every m  iff 𝔄 accepts w.

This suffices by Equivalence (𝖡𝖺𝗌𝖾). The signature σ will consist of a, z, and propositions cα for every possible cell content α of 𝔄, that is, αΓ(Q×Γ). Additionally, φn and φn will use auxiliary propositions, e.g., to encode counters. The only purpose of χ is to mention the propositions in σ; the main work is done by ψn,ψn,χ.

Figure 2: Computation tree of 𝔄 below some wi (drawn horizontally for space constraints).

To explain the idea, let us consider witnesses , for joint σm-consistency of φn,φn for sufficiently large m. By the properties of ψn,ψn, we find 2n points w0,,w2n1 in depth n in which are bisimilar to a single point w^ in depth n in . Recall that in every wi, we have access to its index i via a counter using propositions b0,,bn. Now, χ is a μ𝖬𝖫-formula with the following properties, see also Figure 2 for illustration.

  • χ enforces the “skeleton” of a computation tree for 𝔄, in which each configuration is modeled by a path of length 2n (using an exponential counter), and in which universal and existential configurations alternate.

  • χ also enforces that each point of the skeleton is labeled with some cell content via σ-propositions cα, but without any synchronization except the initial configuration.

  • χ makes sure that below wi the positions 2ni of successor configurations are coordinated.

The key point is that this enforces (due to bisimilarity) a computation tree below w^ in which, due to the last item above, all positions of configurations are coordinated.

We remark that the hardness also holds when σ is not part of the input: one can reduce separability of φ,φ by 𝖬𝖫σ-formulae to separability of φ,φ by (arbitrary) 𝖬𝖫-formulae.

6.2 Upper Bound for Theorem 22

We show that over models of outdegree at most d, 𝖬𝖫-separability of fixpoint formulae can be solved in doubly exponential time. Let us start with establishing a technical but useful fact. For every language of d-ary trees L𝕋d denote the language:

𝖻𝗂𝗌𝖰𝗎𝗈𝗍(L)={𝕋d|there is 𝒩L and a functional bisimulation Z:𝒩𝖻𝗂𝗌}

of bisimulation quotients of trees from L.

Proposition 24.

For every NPTA 𝒜, an NPTA recognizing 𝖻𝗂𝗌𝖰𝗎𝗈𝗍((𝒜)) can be computed in time exponential in the size of 𝒜.

Proof.

Fix an NPTA 𝒜=(Q,Σ,qI,δ,𝗋𝖺𝗇𝗄). For every 𝕋d, we characterize existence of d-ary 𝒩𝒜 with 𝒩𝖻𝗂𝗌 with the following parity game 𝒢𝖻𝗂𝗌𝖰𝗎𝗈𝗍(,𝒜). The game has the set M×Q as positions. The pair (vI,qI) consisting of the root vI of and qI is the initial position. From a position (v,q) first ve chooses Sδ(q,𝗏𝖺𝗅(c)) and a surjective map h:S{v1,,vk} where {v1,,vk} is the set of children of v. Then dam responds with a choice of pS and the next round starts in position (h(p),p). The game is a parity game: the ranks are inherited from 𝒜 in the sense that the rank of (v,q) equals 𝗋𝖺𝗇𝗄(q). It is easy to show that:

ve wins 𝒢𝖻𝗂𝗌𝖰𝗎𝗈𝗍(,𝒜)𝖻𝗂𝗌𝖰𝗎𝗈𝗍((𝒜)) (3)

for every 𝕋d. Using (3) we prove Proposition 24. It suffices to construct an automaton which accepts iff ve wins 𝒢𝖻𝗂𝗌𝖰𝗎𝗈𝗍(,𝒜). To that end, using standard techniques we encode ve’s positional strategies for 𝒢𝖻𝗂𝗌𝖰𝗎𝗈𝗍(,𝒜) as colorings of with 𝒫(Q×Q) and construct, in time exponential in |Q|, an automaton + recognizing models labelled with such winning positional strategies. We then obtain recognizing 𝖻𝗂𝗌𝖰𝗎𝗈𝗍((𝒜)) by projecting out the additional colors 𝒫(Q×Q) from +.

With the help of Proposition 24 we prove Theorem 22. Fix d, μ𝖬𝖫-formulae φ and φ and signature σ. By Equivalence (𝖡𝖺𝗌𝖾), it suffices to check if φ and φ are jointly σn-consistent over 𝕋d for every n. However, unlike with definability or in the binary case, we cannot conclude joint σn-consistency from joint σn-consistency. Instead, we use Proposition 24 to directly decide joint σn-consistency for all n. For a language L𝕋d, define the language:

𝖰𝖯𝖫(L)={𝒩𝕋d|there is L, finite prefix 0 of  and Z:0𝖻𝗂𝗌𝒩}

of finite d-ary trees which are bisimulation quotients of finite prefixes of models from L. By Proposition 24 and the closure properties of parity automata, for every 𝒜 one can construct in exponential time an automaton recognizing 𝖰𝖯𝖫((𝒜)).

We prove the upper bound from Theorem 22. Using Theorem 2 compute automata 𝒜,𝒜 accepting σ-reducts of models of φ,φ. Compute , recognizing 𝖰𝖯𝖫((𝒜)) and 𝖰𝖯𝖫((𝒜)). Recall that any two trees are bisimilar iff they have isomorphic bisimulation quotients. It follows that φ,φ admit a 𝖬𝖫σn-separator over 𝕋d iff 𝒜,𝒜 are joint n-consistent iff , are joint n consistent. By Proposition 7, the latter condition holds for all n iff it holds for n=||+||+1 and this can be tested in time polynomial in ||+||. Since 𝒜,𝒜 are exponential, and , are doubly exponential in the size of φ,φ, this gives the upper bound from Theorem 22.

7 Case Study: Graded Modalities

In this section we apply our techniques and results to the case with graded modal operators. Formally, we extend μ𝖬𝖫 with formulae of the shape gψ and gψ, where {,} and the grade g is a natural number. Intuitively, gψ is true in a point w if w has at least g successors satisfying ψ and dually, gψ is true in w if all but at most g successors satisfy ψ [11, 25]. We denote with 𝗀𝗋𝖬𝖫 and 𝗀𝗋μ𝖬𝖫 the extension of 𝖬𝖫 and μ𝖬𝖫, respectively, with such graded modalities. Clearly, for any d, 𝕋d is 𝗀𝗋μ𝖬𝖫-definable by the formula θd=νx.(dx), which is an additional motivation to study 𝗀𝗋𝖬𝖫 and 𝗀𝗋μ𝖬𝖫.

Indeed, using the results and techniques from the previous section one can easily prove that 𝖬𝖫-separability of 𝗀𝗋μ𝖬𝖫-formulae (defined as expected) is 2-ExpTime-complete.

Theorem 25.

𝖬𝖫-separability of 𝗀𝗋μ𝖬𝖫-formulae is 2-ExpTime-complete.

Proof.

For the lower bound, we reduce 𝖬𝖫-separability of μ𝖬𝖫-formulae over 𝕋3 in spirit similar to Lemma 4. Since the former problem is 2-ExpTime-hard by Theorem 22, the latter is as well. Recall the formula θ3 defining 𝕋3. Then, for any μ𝖬𝖫-formulae φ,φ and ψ𝖬𝖫, we have that ψ is an 𝖬𝖫σ-separator of φ,φ over 𝕋3 iff ψ is an 𝖬𝖫σ-separator of φθd,φθd.

Towards the upper bound, suppose φ,φ𝗀𝗋μ𝖬𝖫. Using standard arguments, one can show that φ,φ are 𝖬𝖫-separable over all models iff they are 𝖬𝖫-separable over 𝕋d, where d=g×(|φ|+|φ|) and g is the greatest grade occurring in φ,φ. We then construct NPTA 𝒜,𝒜 equivalent to φ,φ over d-ary trees via (an analogue for 𝗀𝗋μ𝖬𝖫 of) Theorem 2 and proceed with 𝒜,𝒜 as described in the upper bound proof of Theorem 22.

Interestingly, the problem becomes easier if we allow grades in the separating formula.

Theorem 26.

𝗀𝗋𝖬𝖫-separability of 𝗀𝗋μ𝖬𝖫-formulae is ExpTime-complete.

The lower bound follows by the usual reduction from satisfiability. We thus focus on the upper bound. Similarly to the non-graded case, we establish first a model-theoretic characterization, based on the appropriate notion of bisimilarity that characterizes the expressive power of 𝗀𝗋𝖬𝖫 [10]. A relation Z between models is a graded bisimulation if it satisfies (𝖺𝗍𝗈𝗆) and graded variants of the (𝖻𝖺𝖼𝗄) and (𝖿𝗈𝗋𝗍𝗁) conditions of bisimulations. The graded (𝖿𝗈𝗋𝗍𝗁) condition says that if vZw then for every k and pairwise different children v1,,vk of v, there are pairwise different children w1,,wk of w satisfying viZwi for all ik. The graded (𝖻𝖺𝖼𝗄) condition is symmetric. It is a g-graded bisimulation if the graded (𝖿𝗈𝗋𝗍𝗁) and (𝖻𝖺𝖼𝗄) conditions need to be satisfied only for kg. We denote with 𝐠𝐫𝐝 (resp., g) the fact that there is a graded bisimulation (resp., a g-graded bisimulation) between and that relates their roots. Variants with bounded depth n and/or given signature σ are defined and denoted as expected.

Lemma 27.

For every φ,φ𝗀𝗋μ𝖬𝖫 with maximal grade gmax, signature σ, and n, the following are equivalent:

  1. 1.

    φ,φ are not 𝗀𝗋𝖬𝖫σn-separable (over all models).

  2. 2.

    φ,φ are joint 𝐠𝐫𝐝,σn-consistent (over all models).

  3. 3.

    φ,φ are joint σn-consistent (over all models).

  4. 4.

    φ,φ are joint σn-consistent over 𝕋d for d=gmax×(|φ|+|φ|).

Using Lemma 27, one can solve 𝗀𝗋𝖬𝖫-separability of 𝗀𝗋μ𝖬𝖫 formulae in exponential time, following the approach described in Section 3. More precisely, given φ,φ, we construct NPTA 𝒜,𝒜 equivalent to φ,φ over d-ary trees, d as in Lemma 27, and decide whether 𝒜,𝒜 are joint σn-consistent over 𝕋d for all n via Proposition 7.

Let us provide some details on the proof of the central Lemma 27.

Proof.

We show the implications 12341 in turn. The implication 41 is immediate.

For 12, suppose φ,φ are not 𝗀𝗋𝖬𝖫σn-separable. Hence, for every g there is a pair of models gφ and gφ with gg,σng. One can encode with an 𝖥𝖮-sentence θ that two models and are depth-n trees, is a prefix of some +φ and of some +φ. If Z is a fresh binary symbol, then it is also possible to encode with an (infinite) set T of 𝖥𝖮-sentences that Z is a graded bisimulation between and . Every finite fragment of {θ}T only mentions finitely many grades and hence by assumption is satisfiable. Thus, by compactness of 𝖥𝖮, the entire {θ}T is satisfiable. This gives us 𝐠𝐫𝐝,σn with extensions +φ and +φ.

For 23, fix witnesses , of joint 𝐠𝐫𝐝,σn-consistency, that is, 𝐠𝐫𝐝,σn and there are extensions +,+ of , with +φ and +φ. By the Löwenheim-Skolem property of 𝖥𝖮 we may assume that both models are at most countable. It remains to apply the known fact that countable trees 𝒩 and 𝒩 satisfy 𝒩𝐠𝐫𝐝𝒩 iff 𝒩 and 𝒩 are isomorphic. For the sake of completeness, we add a brief justification of this latter statement. Assume w𝒩 and w𝒩 with respective children w1,w2,=w¯ and w1,w2,=w¯ such that w𝐠𝐫𝐝w. For every 𝐠𝐫𝐝-equivalence class X of w¯ the corresponding equivalence class {wi|jk.wj𝐠𝐫𝐝wi}=X has the same cardinality as X. This is immediate for finite X, and for infinite X it follows because in countable models every two infinite subsets have the same cardinality. This allows us to inductively pick a bijective subrelation Z of 𝐠𝐫𝐝 between 𝒩 and 𝒩 which is still a graded bisimulation.

For 34, fix witnesses , of joint σn-consistency, that is, σn and there are extensions +,+ of , with +φ and +φ. We trim + and + so that the outdegree becomes at most d. Without loosing generality we assume that the prefixes of + and + are not only isomorphic but identical. The semantics of every ψμ𝖬𝖫 in a model 𝒩 is captured by a parity game whose positions are N×𝖲𝗎𝖻𝖥𝗈𝗋(ψ). We extend the definition of the game to μ𝖬𝖫𝐠𝐫𝐝. The set of positions N×𝖲𝗎𝖻𝖥𝗈𝗋(ψ) and the winning condition are defined as in the classical case, and so are the moves for all the positions with topmost connective other than the graded modalities. In the classical game, from (v,θ) ve chooses a child v of v and the next position is (v,θ). In (v,kθ), first ve chooses a subset v1,,vk of size k of children of v, then dam chooses one of these children vi and the next round starts at (vi,θ). Dually, in (v,kθ) first ve picks a subset v1,,vk of at most k v’s children, then dam responds with a choice of some v not in v1,,vk and the next position is (v,θ). It is tedious but straightforward to check that ve wins the game from v,ψ iff ψ is true at v, as in the classical case. Note that if we take a submodel 𝒩0 of 𝒩 which contains at least the root and all -witnesses (that is, points chosen by a winning strategy ζ in for positions of shape (v,kθ)) then (the restriction of) ζ to 𝒩0 is a winning strategy for 𝒢(𝒩0,ψ).

Let ζ and ζ be positional winning strategies for ve in the semantic games 𝒢(+,φ) and 𝒢(+,φ). We take submodel 0φ of + as follows. In the n-prefix we take the root and all -witnesses for both ζ and ζ. In the rest of the model we only take -witnesses for ζ. A submodel 0 of + is defined symmetrically. It follows that 0φ and 0φ.

Recall that g is the maximal grade appearing in φ and φ. Since the respective sets of positions of 𝒢(+,φ) and 𝒢(+,φ) are M+×𝖲𝗎𝖻𝖥𝗈𝗋(φ) and M+×𝖲𝗎𝖻𝖥𝗈𝗋(φ), for every point v there are at most g×|φ| -witnesses chosen by ζ from a position which has v on the first coordinate. Consequently, the outdegree of 0 and 0 is not greater than d=g×(|φ|+|φ|). This proves Lemma 27.

8 Conclusion

We have presented an in-depth study of modal separation of μ𝖬𝖫-formulae over different classes of structures. For us, the most interesting results are the differences that are obtained over classes of bounded outdegree for different bounds d=1, d=2, d3. Without much effort our results on trees of bounded outdegrees can be transferred to infinite words and to ranked trees, via reductions similar to Lemma 4.

Throughout the paper we used the simplest possible measure of formula size: the length of a formula written as a string. Alternative more succinct measures, such as the number of non-isomorphic subformulae (DAG-size), are also interesting. Thus, a natural question is to what extent our results depend on the choice of size measure. In principle, using a more succinct measure makes the problems of definability and separability harder. However, all our decision procedures, with an exception of Theorem 21, are automata-based. Consequently, these procedures carry over with unchanged complexity to any size measure for which the translation from logic to nondeterministic automata has the same complexity as in Theorem 2. In the remaining case of Theorem 21 a weaker assumption suffices: the modal depth of a formula is at most polynomial in its size. Both the mentioned assumptions are arguably modest.

A place where the choice of size measure matters a little more is the construction of modal definitions and separators. In the cases of unrestricted, unary (𝕋1), and high outdegree models (𝕋d for d3) the constructed formulae have DAG-size essentially the same as size: doubly, singly, and triply exponential, respectively. Interestingly, however, in the binary case 𝕋2 our formulae have only singly exponential DAG-size, which is easily seen to be optimal and contrasts with their doubly exponential size. This demonstrates that the lower bounds for size of modal definitions over 𝕋2 cannot work for DAG-size. The same lower bound construction fails for DAG-size over unrestricted models, although there the exact DAG-size complexity of optimal separators remains unknown.

We mention some interesting open problems. First, the relative succinctness of μ𝖬𝖫 over 𝖬𝖫 is to the best of our knowledge open in the setting with only one accessibility relation. Second, as we have mentioned in Section 3, the separators we compute are not necessarily the logically strongest ones. The logically strongest separators of φ,φ are precisely the 𝖬𝖫-uniform consequences of φ (if they exist) and are a natural object of study. Clearly, modal definability of φ is a sufficient condition, but not a necessary one. Let φ=ψ¬θ and φ=ψ for some ψ𝖬𝖫. Then φ is not equivalent to a modal formula, but ψ is a strongest separator. In the context of 𝗀𝗋μ𝖬𝖫, open questions are 𝖬𝖫-definability (and separability) and μ𝖬𝖫-definability (and separability) of 𝗀𝗋μ𝖬𝖫-formulae. We conjecture them to be easier than 2-ExpTime. Finally, let us mention that definability of μ𝖬𝖫-formulae by safety formulae has been studied in [22]. It would be natural to investigate separability there as well.

References

  • [1] Alessandro Artale, Jean Christoph Jung, Andrea Mazzullo, Ana Ozaki, and Frank Wolter. Living without Beth and Craig: Definitions and interpolants in description and modal logics with nominals and role inclusions. ACM Trans. Comput. Log., 24(4):34:1–34:51, 2023. doi:10.1145/3597301.
  • [2] Franz Baader, Ian Horrocks, Carsten Lutz, and Ulrike Sattler. An Introduction to Description Logic. Cambridge University Press, 2017. URL: http://www.cambridge.org/de/academic/subjects/computer-science/knowledge-management-databases-and-data-mining/introduction-description-logic?format=PB#17zVGeWD2TZUeu6s.97.
  • [3] Christel Baier and Joost-Pieter Katoen. Principles of model checking. MIT Press, 2008.
  • [4] Fabio Bellissima. On the lattice of extensions of the modal logics KAltn. Arch. Math. Log., 27(2):107–114, 1988. doi:10.1007/BF01620760.
  • [5] Michael Benedikt, Balder ten Cate, Thomas Colcombet, and Michael Vanden Boom. The complexity of boundedness for guarded logics. In 30th Annual ACM/IEEE Symposium on Logic in Computer Science, LICS, pages 293–304. IEEE Computer Society, 2015. doi:10.1109/LICS.2015.36.
  • [6] Achim Blumensath, Martin Otto, and Mark Weyer. Decidability results for the boundedness problem. Log. Methods Comput. Sci., 10(3), 2014. doi:10.2168/LMCS-10(3:2)2014.
  • [7] Mikołaj Bojańczyk and Wojciech Czerwiński. Automata Toolbox. University of Warsaw, 2018. URL: https://www.mimuw.edu.pl/~bojan/papers/toolbox.pdf.
  • [8] Ashok K. Chandra, Dexter Kozen, and Larry J. Stockmeyer. Alternation. J. ACM, 28(1):114–133, 1981. doi:10.1145/322234.322243.
  • [9] Sang Cho and Dung T. Huynh. Finite-automaton aperiodicity is PSpace-complete. Theor. Comput. Sci., 88(1):99–116, 1991. doi:10.1016/0304-3975(91)90075-D.
  • [10] Maarten de Rijke. A note on graded modal logic. Stud Logica, 64(2):271–283, 2000. doi:10.1023/A:1005245900406.
  • [11] Kit Fine. In so many possible worlds. Notre Dame J. Formal Log., 13(4):516–520, 1972. doi:10.1305/NDJFL/1093890715.
  • [12] Michael J. Fischer and Richard E. Ladner. Propositional dynamic logic of regular programs. J. Comput. Syst. Sci., 18(2):194–211, 1979. doi:10.1016/0022-0000(79)90046-1.
  • [13] Tim French, Wiebe van der Hoek, Petar Iliev, and Barteld P. Kooi. On the succinctness of some modal logics. Artif. Intell., 197:56–85, 2013. doi:10.1016/j.artint.2013.02.003.
  • [14] Martin Fürer. The computational complexity of the unconstrained limited domino problem (with implications for logical decision problems). In Logic and Machines: Decision Problems and Complexity, Proceedings of the Symposium ”Rekursive Kombinatorik”, volume 171 of Lecture Notes in Computer Science, pages 312–319. Springer, 1983. doi:10.1007/3-540-13331-3_48.
  • [15] Dov M. Gabbay. Craig’s interpolation theorem for modal logics. In Conference in Mathematical Logic — London ’70, pages 111–127, Berlin, Heidelberg, 1972. Springer Berlin Heidelberg.
  • [16] Gerd G. Hillebrand, Paris C. Kanellakis, Harry G. Mairson, and Moshe Y. Vardi. Undecidable boundedness problems for datalog programs. J. Log. Program., 25(2):163–190, 1995. doi:10.1016/0743-1066(95)00051-K.
  • [17] Jean Christoph Jung and Jędrzej Kołodziejski. Modal separability of fixpoint formulae. In Proceedings of the 37th International Workshop on Description Logics (DL 2024), volume 3739 of CEUR Workshop Proceedings. CEUR-WS.org, 2024. URL: https://ceur-ws.org/Vol-3739/paper-5.pdf.
  • [18] Jean Christoph Jung and Frank Wolter. Living without Beth and Craig: Definitions and interpolants in the guarded and two-variable fragments. In Proceedings of Annual ACM/IEEE Symposium on Logic in Computer Science (LICS), pages 1–14. IEEE, 2021. doi:10.1109/LICS52264.2021.9470585.
  • [19] Eryk Kopczynski. Invisible pushdown languages. In Proceedings of the 31st Annual ACM/IEEE Symposium on Logic in Computer Science (LICS), pages 867–872. ACM, 2016. doi:10.1145/2933575.2933579.
  • [20] Dexter Kozen. Results on the propositional mu-calculus. Theor. Comput. Sci., 27:333–354, 1983. doi:10.1016/0304-3975(82)90125-6.
  • [21] Louwe Kuijer, Tony Tan, Frank Wolter, and Michael Zakharyaschev. Separating counting from non-counting in fragments of two-variable first-order logic (extended abstract). In Proc. of DL 2024, 2024.
  • [22] Karoliina Lehtinen and Sandra Quickert. Deciding the first levels of the modal mu alternation hierarchy by formula construction. In Proceedings of Annual Conference on Computer Science Logic CSL, volume 41 of LIPIcs, pages 457–471. Schloss Dagstuhl – Leibniz-Zentrum für Informatik, 2015. doi:10.4230/LIPICS.CSL.2015.457.
  • [23] Christof Löding and Christopher Spinrath. Decision problems for subclasses of rational relations over finite and infinite words. Discrete Mathematics & Theoretical Computer Science, Vol. 21 no. 3, January 2019. doi:10.23638/DMTCS-21-3-4.
  • [24] Martin Otto. Eliminating recursion in the μ-calculus. In Proceedings of 16th Annual Symposium on Theoretical Aspects of Computer Science (STACS), volume 1563 of Lecture Notes in Computer Science, pages 531–540. Springer, 1999. doi:10.1007/3-540-49116-3_50.
  • [25] Martin Otto. Graded modal logic and counting bisimulation. CoRR, abs/1910.00039, 2019. arXiv:1910.00039.
  • [26] Thomas Place and Marc Zeitoun. Separating regular languages with first-order logic. Log. Methods Comput. Sci., 12(1), 2016. doi:10.2168/LMCS-12(1:5)2016.
  • [27] Vaughan R. Pratt. A decidable mu-calculus: Preliminary report. In Proceedings of 22nd Annual Symposium on Foundations of Computer Science (FOCS), pages 421–427. IEEE Computer Society, 1981. doi:10.1109/SFCS.1981.4.
  • [28] Abraham Robinson. A result on consistency and its application to the theory of definition. Journal of Symbolic Logic, 25(2):174–174, 1960. doi:10.2307/2964240.
  • [29] Marcel Paul Schützenberger. On finite monoids having only trivial subgroups. Inf. Control., 8(2):190–194, 1965. doi:10.1016/S0019-9958(65)90108-7.
  • [30] A. Prasad Sistla and Edmund M. Clarke. The complexity of propositional linear temporal logics. J. ACM, 32(3):733–749, 1985. doi:10.1145/3828.3837.
  • [31] Moshe Y. Vardi. Reasoning about the past with two-way automata. In Proceedings of International Colloquium Automata, Languages and Programming (ICALP), volume 1443 of Lecture Notes in Computer Science, pages 628–641. Springer, 1998. doi:10.1007/BFB0055090.
  • [32] Yde Venema. Lectures on the modal μ-calculus, 2020.