S2S (mathematics)

From HandWiki

In mathematics, S2S is the monadic second order theory with two successors. It is one of the most expressive natural decidable theories known, with many decidable theories interpretable in S2S. Its decidability was proved by Rabin in 1969.[1]

Basic properties

The first order objects of S2S are finite binary strings. The second order objects are arbitrary sets (or unary predicates) of finite binary strings. S2S has functions ss0 and ss1 on strings, and predicate sS (equivalently, S(s)) meaning string s belongs to set S.

Some properties and conventions:

  • By default, lowercase letters refer to first order objects, and uppercase to second order objects.
  • The inclusion of sets makes S2S second order, with "monadic" indicating absence of k-ary predicate variables for k>1.
  • Concatenation of strings s and t is denoted by st, and is not generally available in S2S, not even s→0s. The prefix relation between strings is definable.
  • Equality is primitive, or it can be defined as s = t ⇔ ∀S (S(s) ⇔ S(t)) and S = T ⇔ ∀s (S(s) ⇔ T(s)).
  • In place of strings, one can use (for example) natural numbers with n→2n+1 and n→2n+2 but no other operations.
  • The set of all binary strings is denoted by {0,1}*, using Kleene star.
  • Arbitrary subsets of {0,1}* are sometimes identified with trees, specifically as a {0,1}-labeled tree {0,1}*; {0,1}* forms a complete infinite binary tree.
  • For formula complexity, the prefix relation on strings is typically treated as first order. Without it, not all formulas would be equivalent to Δ12 formulas.[2]
  • For properties expressible in S2S (viewing the set of all binary strings as a tree), for each node, only O(1) bits can be communicated between the left subtree and the right subtree and the rest (see communication complexity).
  • For a fixed k, a function from strings to k (i.e. natural numbers below k) can be encoded by a single set. Moreover, s,ts01t where t doubles every character of t is injective, and s ⇒ {s01t: t∈{0,1}*} is S2S definable. By contrast, by a communication complexity argument, in S1S (below) a pair of sets is not encodable by a single set.

Weakenings of S2S: Weak S2S (WS2S) requires all sets to be finite (note that finiteness is expressible in S2S using Kőnig's lemma). S1S can be obtained by requiring that '1' does not appear in strings, and WS1S also requires finiteness. Even WS1S can interpret Presburger arithmetic with a predicate for powers of 2, as sets can be used to represent unbounded binary numbers with definable addition.

Decision complexity

S2S is decidable, and each of S2S, S1S, WS2S, WS1S has a nonelementary decision complexity corresponding to a linearly growing stack of exponentials. For the lower bound, it suffices to consider Σ11 WS1S sentences. A single second order quantifier can be used to propose an arithmetic (or other) computation, which can be verified using first order quantifiers if we can test which numbers are equal. For this, if we appropriately encode numbers 1..m, we can encode a number with binary representation i1i2...im as i1 1 i2 2 ... im m, preceded by a guard. By merging testing of guards and reusing variable names, the number of bits is linear in the number of exponentials. For the upper bound, using the decision procedure (below), sentences with k-fold quantifier alternation can decided in time corresponding to k+O(1)-fold exponentiation of the sentence length (with uniform constants).

Axiomatization

WS2S can be axiomatized through certain basic properties plus induction schema.[3]

S2S can be partially axiomatized by:
(1) ∃!st ( t0≠st1≠s) (empty string, denoted by ε; ∃!s means "there is unique s")
(2) ∀s,ti∈{0,1} ∀j∈{0,1} (si=tjs=ti=j) (the use of i and j is an abbreviation; for i=j, 0 does not equal 1)
(3) ∀S (S(ε) ∧ ∀s (S(s) ⇒ S(s0) ∧ S(s1))⇒ ∀s S(s)) (induction)
(4) ∃Ss (S(s) ⇔ φ(s)) (S not free in φ)

(4) is the comprehension schema over formulas φ, which always holds for second order logic. As usual, if φ has free variables not shown, we take the universal closure of the axiom. If equality is primitive for predicates, one also adds extensionality S=T ⇔ ∀s (S(s) ⇔ T(s)). Since we have comprehension, induction can be a single statement rather than a schema.

The analogous axiomatization of S1S is complete.[4] However, for S2S, completeness is open (as of 2021). While S1S has uniformization, there is no S2S definable (even allowing parameters) choice function that given a non-empty set S returns an element of S,[5] and comprehension schemas are commonly augmented with various forms of the axiom of choice. However, (1)-(4) is complete when extended with a determinacy schema for certain parity games.[6]

S2S can also be axiomatized by Π13 sentences (using the prefix relation on strings as a primitive). However, it is not finitely axiomatizable, nor can it be axiomatized by Σ13 sentences even if we add induction schema and a finite set of other sentences (this follows from its connection to Π12-CA0).

Theories related to S2S

For every finite k, the monadic second order (MSO) theory of countable graphs with treewidthk (and a corresponding tree decomposition) is interpretable in S2S (see Courcelle's theorem). For example, the MSO theory of trees (as graphs) or of series-parallel graphs is decidable. Here (i.e. for bounded tree width), we can also interpret the finiteness quantifier for a set of vertices (or edges), and also count vertices (or edges) in a set modulo a fixed integer. Allowing uncountable graphs does not change the theory. Also, for comparison, S1S can interpret connected graphs of bounded pathwidth.

By contrast, for every set of graphs of unbounded treewidth, its existential (i.e. Σ11) MSO theory is undecidable if we allow predicates on both vertices and edges. Thus, in a sense, decidability of S2S is the best possible. Graphs with unbounded treewidth have large grid minors, which can be used to simulate a Turing machine.

By reduction to S2S, the MSO theory of countable orders is decidable, as is the MSO theory of countable trees with their Kleene–Brouwer orders. However, the MSO theory of ([math]\displaystyle{ \mathbb{R} }[/math], <) is undecidable.[7][8] The MSO theory of ordinals <ω2 is decidable; decidability for ω2 is independent of ZFC (assuming Con(ZFC + weakly compact cardinal)).[9] Also, an ordinal is definable using monadic second order logic on ordinals iff it can be obtained obtained from definable regular cardinals by ordinal addition and multiplication.[10]

S2S is useful for decidability of certain modal logics, with Kripke semantics naturally leading to trees.

S2S+U (or just S1S+U) is undecidable if U is the unbounding quantifier — UX Φ(X) iff Φ(X) holds for some arbitrarily large finite X.[11] However, WS2S+U, even with quantification over infinite paths, is decidable, even with S2S subformulas that do not contain U.[12]

Formula complexity

A set of binary strings is definable in S2S iff it is regular (i.e. forms a regular language). In S1S, a (unary) predicate on sets is (parameter-free) definable iff it is an ω-regular language. For S2S, for formulas that use their free variables only on strings not containing a 1, the expressiveness is the same as for S1S.

For every S2S formula φ(S1,...,Sk), (with k free variables) and finite tree of binary strings T, φ(S1∩T,...,Sk∩T) can be computed in time linear in |T| (see Courcelle's theorem), but as noted above, the overhead can be iterated exponential in the formula size (more precisely, the time is [math]\displaystyle{ O(|T|k)+2_{O(|\phi|)}^2 }[/math]).

For S1S, every formula is equivalent to a Δ11 formula, and to a boolean combination of Π02 arithmetic formulas. Moreover, every S1S formula is equivalent to acceptance by a corresponding ω-automaton of the parameters of the formula. The automaton can be a deterministic parity automaton: A parity automaton has an integer priority for each state, and accepts iff the highest priority seen infinitely often is odd (alternatively, even).

For S2S, using tree automata (below), every formula is equivalent to a Δ12 formula. Moreover, every S2S formula is equivalent to a formula with just four quantifiers, ∃STst ... (assuming that our formalization has both the prefix relation and the successor functions). For S1S, three quantifiers (∃Sst) suffice, and for WS2S and WS1S, two quantifiers (∃St) suffice; the prefix relation is not needed here for WS2S and WS1S.

However, with free second order variables, not every S2S formula can be expressed in second order arithmetic through just Π11 transfinite recursion (see reverse mathematics). RCA0 + (schema) {τ: τ is a true S2S sentence} is equivalent to (schema) {τ: τ is a Π13 sentence provable in Π12-CA0 }.[13][14] Over a base theory, the schemas are equivalent to (schema over k) ∀S⊆ω ∃α1<...<αk Lα1(S) ≺Σ1 ... ≺Σ1 Lαk(S) where L is the constructible universe (see also large countable ordinal). Due to limited induction, Π12-CA0 does not prove that all true (under the standard decision procedure) Π13 S2S statements are actually true even though each such sentence is provable Π12-CA0.

Moreover, given sets of binary strings S and T, the following are equivalent:
(1) T is S2S definable from some set of binary strings polynomial time computable from S.
(2) T can be computed from the set of winning positions for some game whose payoff is a finite boolean combination of Π02(S) sets.
(3) T can be defined from S in arithmetic μ-calculus (arithmetic formulas + least fixed-point logic)
(4) T is in the least β-model (i.e. an ω-model whose set-theoretic counterpart is transitive) containing S and satisfying all Π13 consequences of in Π12-CA0.

Proof sketch:

See [13] and,[15] but briefly the proof runs as follows. (1)⇒(2) follows from the below decidability proof using tree automata. (2)⇒(1) follows by converting the game associated with a binary string s into a tree parity game with a fixed number of priorities and then merging these trees into a single tree (the binary trees can be merged here using s,ts01t where t doubles every character of t). The below determinacy proof (in the decidability section) also leads to (2)⇒(3). Π12-CA0 proves Δ12 monotonic induction, so (3)⇒(4).

For (3)⇒(2), define a game where player 1 attempts to show that the desired element s is inside the least fixed point. Player 1 gradually labels elements including s with rational numbers, intended to correspond to ordinal stages of the monotonic induction (any countable ordinal is embeddable into [math]\displaystyle{ \mathbb{Q} }[/math]). Player 2 plays elements with strictly descending labels (and he can pass) and wins iff the sequence is infinite or player 2 wins the last auxiliary game. In the auxiliary game, player 1 attempts to show that the last element picked by player 2 is a valid inductive step using elements with smaller labels. Now, if s is not in the least fixed-point, then the set of labels is ill-founded, or an inductive step is wrong, and (using monotonicity) this can be picked up by player 2. (If player 1 plays a smaller label outside the least fixed point, player 2 can use it (abandoning the auxiliary game), otherwise (using monotonicity) player 2 can use an auxiliary game strategy that assumes that the set of smaller labels in the original game will equal the least fixed point.)

For (4)⇒(3), we use monotonic induction to build an initial segment of the constructible hierarchy above a given real number r. This works as long as each ordinal α is identified by some appropriately expressible property of α so that we can encode α by a natural number and continue. Now, suppose that we built Lα(r) and the inductive step (which uses Lα(r) as a parameter) allows examining Lβ(r). If a new Σ1(L(r),∈,r) fact appears between α and β, we can use it to label α and continue. Otherwise, we get the above Σ1 elementary chains whose length corresponds to the nesting depth of the monotonic inductive definitions.

For the equivalence of RCA0+S2S with {Π13 φ: Π12-CA0⊢φ}, for each k the positional determinacy with k priorities is provable in Π12-CA0, while the rest (in terms of proving S2S sentences) can be done in a weak base theory. Conversely, RCA0+S2S gives us a determinacy schema that gives existence of least fixed points (by a modification of the above (3)⇒(2) and even without requiring positionality; see the reference). In turn, their existence (using (4)⇒(3)) gives the desired Σ1 elementary chains.

Models of S1S and S2S

In addition to the standard model (which is the unique MSO model for S1S and S2S), there are other models for S1S and S2S, which use some rather than all subsets of the domain (see Henkin semantics).

For every S⊆ω, sets recursive in S form an elementary submodel of the standard S1S model, and same for every non-empty collection of subsets of ω closed under Turing join and Turing reducibility.[16]

This follows from relative recursiveness of S1S definable sets plus uniformization:
- φ(s) (as a function of s) can be computed from the parameters of φ and the values of φ(s) for a finite set of s (with its size bounded by the number of states in a deterministic automaton for φ).
- A witness for ∃S φ(S) can be obtained by choosing k and a finite fragment of S of S, and repeatedly extending S such that the highest priority during each extension is k and that the extension can be completed into S satisfying φ without hitting priorities above k (these are permitted only for the initial S). Also, by using lexicographically least shortest choices, there is an S1S formula φ' such that φ'⇒φ and ∃S φ(S) ⇔∃!S φ'(S) (i.e. uniformization; φ may have free variables not shown; φ' depends only on the formula φ).

The minimal model of S2S consists of all regular languages on binary strings. It is an elementary submodel of the standard model, so if an S2S parameter-free definable set of trees is non-empty, then it includes a regular tree. A regular language can also be treated as a regular {0,1}-labeled complete infinite binary tree (identified with predicates on strings). A labeled tree is regular if it can be obtained by unrolling a vertex-labeled finite directed graph with an initial vertex; a (directed) cycle in the graph reachable from the initial vertex gives an infinite tree. With this interpretation and encoding of regular trees, every true S2S sentence may already be provable in elementary function arithmetic. It is non-regular trees that may require nonpredicative comprehension for determinacy (below). There are nonregular (i.e. containing nonregular languages) models of S1S (and presumably S2S) (both with and without standard first order part) with a computable satisfaction relation. However, the set of recursive sets of strings does not form a model of S2S due to failure of comprehension and determinacy.

Decidability of S2S

The proof of decidability is by showing that every formula is equivalent to acceptance by a nondeterministic tree automaton (see tree automaton and infinite-tree automaton). An infinite tree automaton starts at the root and moves up the tree, and accepts iff every tree branch accepts. A nondeterministic tree automaton accepts iff player 1 has a winning strategy, where player 1 chooses an allowed (for the current state and input) pair of new states (p0,p1), while player 2 chooses the branch, with the transition to p0 if 0 is chosen and p1 otherwise. For a co-nondeterministic automaton, all choices are by player 2, while for deterministic, (p0,p1) is fixed by the state and input; and for a game automaton, the two players play a finite game to set the branch and the state. Acceptance on a branch is based on states seen infinitely often on the branch; parity automata are sufficiently general here.

For converting the formulas to automata, the base case is easy, and nondeterminism gives closure under existential quantifiers, so we only need closure under complementation. Using positional determinacy of parity games (which is where we need impredicative comprehension), non-existence of player 1 winning strategy gives a player 2 winning strategy S, with a co-nondeterministic tree automaton verifying its soundness. The automaton can then be made deterministic (which is where we get an exponential increase in the number of states), and thus existence of S corresponds to acceptance by a non-deterministic automaton.

Determinacy: Provably in ZFC, Borel games are determined, and the determinacy proof for boolean combinations of Π02 formulas (with arbitrary real parameters) also gives a strategy here that depends only on the current state and the position in the tree. The proof is by induction on the number of priorities. Assume that there are k priorities, with the highest priority being k, and that k has the right parity for player 2. For each position (tree position + state) assign the least ordinal α (if any) such that player 1 has a winning strategy with all entered (after one or more steps) priority k positions (if any) having labels <α. Player 1 can win if the initial position is labeled: Each time a priority k state is reached, the ordinal is decreased, and moreover in between the decreases, player 1 can use a strategy for k-1 priorities. Player 2 can win if the position is unlabeled: By the determinacy for k-1 priorities, player 2 has a strategy that wins or enters an unlabeled priority k state, in which case player 2 can again use that strategy. To make the strategy positional (by induction on k), when playing the auxiliary game, if two chosen positional strategies lead to the same position, continue with the strategy with the lower α, or for the same α (or for player 2) lower initial position (so we can switch a strategy finitely many times).

Automata determinization: For determinization of co-nondeterministic tree automata, it suffices to consider ω-automata, treating branch choice as input, determinizing the automaton, and using it for the deterministic tree automaton. Note that this does not work for nondeterministic tree automata as the determinization for going left (i.e. ss0) can depend on the contents of the right branch; by contrast to nondeterminism, deterministic tree automata cannot even accept precisely nonempty sets. To determinize a nondeterministic ω-automaton M (for co-nondeterministic, take the complement, noting that deterministic parity automata are closed under complements), we can use a Safra tree with each node storing a set of possible states of M, and node creation and deletion based on reaching high priority states. For details, see [17] or.[18]

Decidability of acceptance: Acceptance by a nondeterministic parity automaton of the empty tree corresponds to a parity game on a finite graph G. Using the above positional (also called memoryless) determinacy, this can be simulated by a finite game that ends when we reach a loop, with the winning condition based on the highest priority state in the loop. A clever optimization gives a quasipolynomial time algorithm,[19] which is polynomial time when the number of priorities is small enough (which occurs commonly in practice).

Theory of trees: For decidability of MSO logic on trees (i.e. graphs that are trees), even with finiteness and modular counting quantifiers for first order objects, we can embed countable trees into the complete binary tree and use the decidability of S2S. For example, for a node s, we can represent its children by s1, s01, s001, and so on. For uncountable trees, we can use Shelah-Stup theorem (below). We can also add a predicate for a set first order objects having cardinality ω1, and the predicate for cardinality ω2, and so on for infinite regular cardinals. Graphs of bounded tree width are interpretable using trees, and without predicates over edges this also applies to graphs of bounded clique width.

Combining S2S with other decidable theories

Tree extensions of monadic theories: By Shelah-Stup theorem,[20][21] if a monadic relational model M is decidable, then so is its tree counterpart. For example, (modulo choice of formalization) S2S is the tree counterpart of {0,1}. In the tree counterpart, the first order objects are finite sequences of elements of M ordered by extension, and an M-relation Pi is mapped to Pi'(vd1,...,vdk) ⇔ Pi(d1,...,dk) with Pi' false otherwise (djM, and v is a (possibly empty) sequence of elements of M). The proof is similar to the S2S decidability proof. At each step, a (nondeterministic) automaton gets a tuple of M objects (possibly second order) as input, and an M formula determines which state transitions are permitted. Player 1 (as above) chooses a mapping child⇒state that is permitted by the formula (given the current state), and player 2 chooses the child (of the node) to continue. To witness rejection by a non-deterministic automaton, for each (node, state) pick a set of (child, state) pairs such that for every choice, at least one of the pairs is hit, and such that all the resulting paths lead to rejection.

Combining a monadic theory with a first order theory: Feferman–Vaught theorem extends/applies as follows. If M is an MSO model and N is a first order model, then M remains decidable relative to a (Theory(M), Theory(N)) oracle even if M is augmented with all functions MN where M is identified with its first objects, and for each sM we use a disjoint copy of N, with the language modified accordingly. For example, if N is ([math]\displaystyle{ \mathbb{R} }[/math],0,+,⋅), we can state ∀(function f) ∀srNs f(s) +Ns r = 0Ns. If M is S2S (or more generally, the tree counterpart of some monadic model), the automata can now use N-formulas, and thereby convert f:MNk into a tuple of M sets. Disjointness is necessary as otherwise for every infinite N with equality, the extended S2S or just WS1S is undecidable. Also, for a (possibly incomplete) theory T, the theory TM of M-products of T is decidable relative to a (Theory(M), T) oracle, where a model of TM uses an arbitrary disjoint model Ns of T for each sM (as above, M is an MSO model; Theory(Ns) may depend on s). The proof is by induction on formula complexity. Let vs be the list of free Ns variables, including f(s) if function f is free. By induction, one shows that vs is only used through a finite set of N-formulas with |vs| free variables. Thus, we can quantify over all possible outcomes by using N (or T) to answer what is possible, and given a list possibilities (or constraints), formulate a corresponding sentence in M.

Coding into extensions of S2S: Every decidable predicate on strings can be encoded (with linear time encoding and decoding) for decidability of S2S (even with the extensions above) together with the encoded predicate. Proof: Given a nondeterministic infinite tree automaton, we can partition the set of finite binary labeled trees (having labels over which the automaton can operate) into finitely many classes such that if a complete infinite binary tree can be composed of same-class trees, acceptance depends only on the class and the initial state (i.e. state the automaton enters the tree). (Note a rough similarity with the pumping lemma.) For example (for a parity automaton), assign trees to the same class if they have the same predicate that given initial_state and set Q of (state, highest_priority_reached) pairs returns whether player 1 (i.e. nondeterminism) can simultaneously force all branches to correspond to elements of Q. Now, for each k, pick a finite set of trees (suitable for coding) that belong to the same class for automata 1-k, with the choice of class consistent across k. To encode a predicate, encode some bits using k=1, then more bits using k=2, and so on.

References

  1. Rabin, Michael (1969). "Decidability of second-order theories and automata on infinite trees". Transactions of the American Mathematical Society 141. https://www.ams.org/journals/tran/1969-141-00/S0002-9947-1969-0246760-1/S0002-9947-1969-0246760-1.pdf. 
  2. Janin, David; Lenzi, Giacomo. "On the Structure of the Monadic Logic of the Binary Tree". MFCS 1999. doi:10.1007/3-540-48340-3_28. https://hal.archives-ouvertes.fr/hal-00676277. 
  3. Siefkes, Dirk (1971), An axiom system for the weak monadic second order theory of two successors, https://docs.lib.purdue.edu/cgi/viewcontent.cgi?article=1477&context=cstech 
  4. Riba, Colin (2012). "A model theoretic proof of completeness of an axiomatization of monadic second-order logic on infinite words". TCS 2012. doi:10.1007/978-3-642-33475-7_22. https://link.springer.com/content/pdf/10.1007%2F978-3-642-33475-7_22.pdf. 
  5. Carayol, Arnaud; Löding, Christof (2007), "MSO on the Infinite Binary Tree: Choice and Order", Computer Science Logic, Lecture Notes in Computer Science, 4646, pp. 161–176, doi:10.1007/978-3-540-74915-8_15, ISBN 978-3-540-74914-1, https://hal-upec-upem.archives-ouvertes.fr/hal-00620169/file/csl07.pdf 
  6. Das, Anupam; Riba, Colin (2020). "A functional (monadic) second-order theory of infinite trees". Logical Methods in Computer Science 16 (4). doi:10.23638/LMCS-16(4:6)2020.  (A preliminary 2015 version erroneously claimed proof of completeness without the determinacy schema.)
  7. Gurevich, Yuri; Shelah, Saharon (1984). "The monadic theory and the "next world"". Israel Journal of Mathematics 49 (1–3): 55–68. doi:10.1007/BF02760646. 
  8. "What is the Turing degree of the monadic theory of the real line?". MathOverflow. https://mathoverflow.net/questions/385530/what-is-the-turing-degree-of-the-monadic-theory-of-the-real-line. 
  9. Gurevich, Yuri; Magidor, Menachem; Shelah, Saharon (1993). "The monadic theory of ω2". The Journal of Symbolic Logic 48 (2): 387–398. doi:10.2307/2273556. https://shelah.logic.at/files/95215/141.pdf. 
  10. Neeman, Itay (2008), "Monadic definability of ordinals", Computational Prospects of Infinity, Lecture Notes Series, Institute for Mathematical Sciences, National University of Singapore, 15, pp. 193–205, doi:10.1142/9789812796554_0010, ISBN 978-981-279-654-7, https://www.math.ucla.edu/~ineeman/monadic-def.pdf 
  11. Bojańczyk, Mikołaj; Parys, Paweł; Toruńczyk, Szymon (2015), The MSO+U theory of (N, <) is undecidable 
  12. Bojańczyk, Mikołaj (2014), Weak MSO+U with path quantifiers over infinite trees 
  13. 13.0 13.1 Kołodziejczyk, Leszek; Michalewski, Henryk (2016). "How unprovable is Rabin's decidability theorem?". LICS '16: 31st Annual ACM/IEEE Symposium on Logic in Computer Science. 
  14. Kołodziejczyk, Leszek (October 19, 2015). "Question on Decidability of S2S". FOM. https://cs.nyu.edu/pipermail/fom/2015-October/019257.html. 
  15. Heinatsch, Christoph; Möllerfeld, Michael (2010). "The determinacy strength of Π12-comprehension". Annals of Pure and Applied Logic 161 (12): 1462–1470. doi:10.1016/j.apal.2010.04.012. https://core.ac.uk/download/pdf/81981008.pdf. 
  16. Kołodziejczyk, Leszek; Michalewski, Henryk; Pradic, Pierre; Skrzypczak, Michał (2019). "The logical strength of Büchi's decidability theorem". Logical Methods in Computer Science 15 (2): 16:1–16:31. https://lmcs.episciences.org/5503/. 
  17. Piterman, Nir (2006). "From Nondeterministic Buchi and Streett Automata to Deterministic Parity Automata". 21st Annual IEEE Symposium on Logic in Computer Science (LICS'06). pp. 255–264. doi:10.1109/LICS.2006.28. 
  18. Löding, Christof; Pirogov, Anton. "Determinization of Büchi Automata: Unifying the Approaches of Safra and Muller-Schupp". ICALP 2019. 
  19. Calude, Cristian; Jain, Sanjay; Khoussainov, Bakhadyr; Li, Wei; Stephan, Frank. "Deciding parity games in quasipolynomial time". STOC 2017. https://researchspace.auckland.ac.nz/bitstream/handle/2292/31757/500Cris.pdf. 
  20. Shelah, Saharon (Nov 1975). "Monadic theory of order". Annals of Mathematics 102 (3): 379–419. doi:10.2307/1971037. https://shelah.logic.at/files/213042/42.pdf. 
  21. "The generalization of Shelah–Stup theorem". https://www.mccme.ru/shen/muchnik-memorial/materials/publications/tree_str.pdf. 

Additional reference:
Weyer, Mark (2002). "Decidability of S1S and S2S". Automata, Logics, and Infinite Games. Lecture Notes in Computer Science. 2500. Springer. pp. 207–230. doi:10.1007/3-540-36387-4_12. ISBN 978-3-540-00388-5. https://link.springer.com/chapter/10.1007/3-540-36387-4_12.