Fast LTL to Büchi Automata Translation

Size: px
Start display at page:

Download "Fast LTL to Büchi Automata Translation"

Transcription

1 (LTL2BA) April 19, 2013

2 (LTL2BA) Table of contents 1 (LTL2BA) 2 Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA 3

3 (LTL2BA) (LTL2BA) (TGBA)

4 (LTL2BA) Very Weak Alternating Automata (VWAA) Definition 6: A co-büchi very weak alternating co-büchi automaton is a five tuple A = (Q, Σ, δ, I, F) - Q is the set of states - Let Q be the set of conjunctions of elements of Q. The empty conjunction is denoted by tt. We identity Q with 2 Q in the following - Σ is the alphabet, and we let Σ = 2 Σ - δ : Q 2 Σ xq - I Q is the set of initial states - F Q is the set of final states (co-büchi) - There exists a partial order on Q such that q Q, all the states appearing in δ(q) are lower or equal to q very weak

5 (LTL2BA) Figure: Automaton A θ. Some states (right) are unaccessible, they will be removed. I = {GFp F(q G r)}, δ(p) = {(Σ p, tt)} where Σ p = {a Σ p a}, δ(gfp) = {(Σ p, GFp), (Σ, GFp Fp)}.

6 (LTL2BA) A run σ of A on a word u 0 u 1... Σ ω is labeled DAG(V, E, λ) - V is partitioned in V i with E V i xv i+1 i=0 - λ: V Q is the labeling function i=0 - λ(v 0 ) I and x V i, (a, e) δ(λ(x)), u i a and e = λ(e(x)). A run σ is accepting if any (infinite) branch in σ has only a infinite number of nodes labeled in F (co-büchi acceptance condition).

7 (LTL2BA) Figure: Automaton A θ. Some states (right) are unaccessible, they will be removed. Figure: Example of an accepting run of the automaton A θ.

8 (LTL2BA) Definition 7: - For J 1 J 2 2 Σ xq : J 1 J2 = (a 1 a 2, e 1 e 2 ) (a 1, e 1 ) J 1 and (a 2, e 2 ) J 2 - Let ψ be an LTL formula in positive normal form. We define ψ by: ψ = {{ψ}} if ψ is a temporal formula ψ 1 ψ 2 = {e 1 e 2 e 1 ψ 1 and e 2 ψ 2 } and ψ 1 ψ 2 = ψ 1 ψ 2

9 (LTL2BA) Let ϕ be an LTL formula on a set Prop. Define the VWAA A ϕ : - Q is the set of temporal subformulae of ψ - Σ = 2 Prop, I = ψ - F is the set of until subformulae of ψ - δ is defined as follows ( extends δ to all subformulae of ϕ) δ(tt) = {(Σ, tt)} δ(p) = {(Σ p, tt)} where Σ p = {a Σ p a} δ( p) = {(Σ p, tt)} where Σ p = Σ\Σ p δ(x ψ) = {(Σ, e) e ψ} δ(ψ 1 ψ 2 ) = (ψ 2 ) ( (ψ 1 ) {(Σ, ψ 1 ψ 2 )}) δ(ψ 1 Rψ 2 ) = (ψ 2 ) ( (ψ 1 ) {(Σ, ψ 1 Rψ 2 )}) (ψ) = δ(ψ) if ψ is a temporal formula (ψ 1 ψ 2 ) = (ψ 1 ) (ψ 2 ) (ψ 1 ψ 2 ) = (ψ 1 ) (ψ 2 )

10 (LTL2BA) Example Let ϕ = (GFp G(q Fr)) - ϕ def = (ff R(ttUp)) (ttu(q (ff R r))) - Transition function (have 10 states totally) δ( r) = {(Σ r, tt)} δ(ff R r) = {(Σ r, ff R r)} δ(q (ff R r)) = (q) (ff R r) = {(Σ r Σ q, ff R r)} δ(ttup) = {(Σ p, tt), (Σ, ttup)}... - Initial state I = ϕ = GFp F(q G r) - Final states F is formula of type ϕ 1 Uϕ 2 = {F(q G r), Fp}

11 (LTL2BA) Transition Based Generalized Büchi Automata (TGBA) Definition 8: A generalized Büchi automaton is a five-tuple G = (Q, Σ, δ, I, T ) where: - Q is the set of states - Σ is the alphabet, and we let Σ 2 Σ - δ : Q 2 Σ xq is the transition function - I Q is the set of initial states - T = {T 1,..., T r } where T j QxΣ xq are the accepting transitions

12 (LTL2BA) Figure: Automaton G Aθ, before (left) and after (right). A run σ of G on word u 0 u 1... Σ ω is a sequence q 0, q 1,... of elements of Q such that q 0 I and i 0, a i Σ such that u i a i and (a i, q i+1 ) δ(q i ). A run σ is accepting if for each 1 j r it uses infinitely many transitions from T j. L(G) is the set of words on which there exists accepting run of G.

13 (LTL2BA) Let A = (Q, Σ, δ, I, F ) be a VWAA with co-büchi acceptance conditions. We define the GBA G A = (Q, Σ, δ, I, T ) where: - Q = 2 Q is identified with conjunctions of states - δ (q 1... q n ) = n δ(q i ) i=1 - δ is the set of -minimal transition of δ where the relation is defined by t t if t = (e,a,e ), t = (e,a,e ), a a, e e, and T T, t T t T - T = {T f f F } where T f = {(e, α, e ) f / e or (β, e ) δ(f ), α β and f / e e }

14 (LTL2BA) Example Find δ (GFp F(q G r)) - δ (GFp F(q G r)) (Σ p, GFp F(q G r)) : T Fp, (Σ p Σ q Σ r, GFp G r) : T Fp, T F(q G r), (Σ, GFp Fp F(q G r)) :, (Σ q Σ r, GFp Fp G r) : T F(q G r) - δ (GFp F(q G r) (Σ p, GFp F(q G r)), (Σ p Σ q Σ r, GFp G r), (Σ, GFp Fp F(q G r)), (Σ q Σ r, GFp Fp G r)

15 (LTL2BA) Example Find δ (GFp Fp G r) - δ (GFp Fp G r) (Σ p Σ r, GFp G r) : T Fp, T F(q G r), (Σ p Σ r, GFp Fp F(q G r)) : T F(q G r), (Σ r, GFp Fp F(q G r)) : T F(q G r) - δ (GFp Fp G r) (Σ p Σ r, GFp G r), (Σ r, GFp Fp F(q G r))

16 (LTL2BA) Büchi Automata (BA) Definition 9: A Büchi automaton is a five-tuple B = (Q, Σ, δ, I, F ) - Q is the set of states - Σ is the alphabet, and we let Σ 2 Σ - δ : Q 2 Σ xq is the transition function - I Q is the set of initial states - F Q is the set of repeated states (Büchi condition) Let G = (Q, Σ, δ, I, F ) be a GBA with T = {T 1,..., T 2 }. We define the BA B G = (Qx{0,..., r}, Σ, δ, Ix{0}, Qx{r}) δ ((q, j)) = {α, (q{, j )) (α, q ) δ(q) and j = next(j, (q, α, q ))}. max{j i r j < k i, t T k }if j r with next(j,t) = max{j < i r 0 < k i, t T k }if j = r

17 (LTL2BA) Figure: Automaton B GAθ after. A run σ of B on a word u 0 u 1... Σ ω is a sequence q 0, q 1,... of elements of Q such that q 0 I and i 0, a i Σ such that u i a i and (a i, q i+1 ) δ(q i ). A run σ is accepting if there exists infinitely many states in F. L(B) is the set of words on which there exists an accepting run of B.

18 (LTL2BA) Example T = {T F(q G r), T Fp } δ(a) = {(Σ p, A), (Σ, A), (Σ p Σ q Σ r, B), (Σ q Σ r, B)} next(0, (A, Σ p, A)) = 0 because T Fp next(0, (A, Σ, A)) = 0 next(0, (Σ p Σ q Σ r, B)) = 2 because T F(q G r), T Fp next(0, (Σ q Σ r, B)) = 1 because T F(q G r) δ (A, 0) = {(Σ p, (A, 0)), (Σ, (A, 0)), (Σ p Σ q Σ r, (B, 2)), (Σ q Σ r, (B, 1))}

19 (LTL2BA) - A state that is not accessible can be removed, - If a transition t 1 implies a transition t 2, then t 2 can be removed. t 1 = (q, a 1, q 1 ) implies t 2 = (q, a 2, q 2 ) if In VWAA: a 2 a 1 and q 1 q 2 In GBA: a 2 a 1, q 1 = q 2 and t T, t 2 T t 1 T In BA: a 2 a 1 and q 1 = q 2 - If two states q 1 and q 2 are equivalent, then they can be merged. q 1 and q 2 are equivalent if In VWAA: δ(q 1 ) = δ(q 2 ) and q 1 F q 2 F In GBA: δ(q 1 ) = δ(q 2 ) and (a, q ) δ(q 1 ), T T, (q 1, a, q ) T (q 2, a, q ) T In BA: δ(q 1 ) = δ(q 2 ) and q 1 F q 2 F

20 (LTL2BA) Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA

21 (LTL2BA) Alternating Formula Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Lemma 1. - Every pure eventuality formula µ satisfies the following: ω Σ ω, u Σ : ω = µ uω = µ (left-append closed languages) - Every pure universality formula ν satisfies the following: ω Σ ω, u Σ : uω = ν ω = ν (suffix closed languages) Lemma 2. - Every alternating formula ε satisfies the following: ω Σ ω, u Σ : ω = ε uω = ε (prefix-invariant languages)

22 (LTL2BA) Alternating Formula Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Definition 10: Let ϕ ranges over general LTL formula. Define classes pure eventuality formula µ, pure universality formula ν, and alternating formula ε - µ ::= Fϕ µ µ µ µ Xµ ϕuµ µrµ Gµ - ν ::= Gϕ ν ν ν µ Xµ νuν ϕrν Fν - ε ::= Gµ Fν ε ε ε ε Xε ϕuε ϕrε Fε Gε Reduction of LTL formula. Let ϕ, ψ range over LTL formula and γ ranges over alternating ones. XϕRXψ X(ϕRψ), ϕuγ γ, Fγ γ, Xγ γ, Xϕ Xψ X(ϕ ψ), ϕrγ γ, Gγ γ

23 (LTL2BA) Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Given an input LTL formula ϕ, an equivalent VWAA is constructed as A ϕ = (Q, Σ, δ, I, F ), where Q, Σ, F are defined as in the original construction, I = {ϕ}

24 (LTL2BA) Example Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Figure: VWAA for (GFa)Ub generate by (a) the translation of LTL2BA, (b) LTL3BA translation with suspension.

25 (LTL2BA) Example Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Let ϕ = (GFa)Ub def = (ff R(ttUa))Ub - δ(ttua) = {(Σ, ttua), (Σ a, tt)} - δ(ff R(ttUa)) = {(Σ a, GFa), (Σ, GFa Fa)} - In LTL2BA: δ((gfa)ub) = (b)u( (GFa) {(Σ, (GFa)Ub)}) = {(Σ b, tt), (Σ a, GFa ((GFa)Ub)), (Σ, GFa Fa ((GFa)Ub))} - In LTL3BA (we have GFa is alternating): δ((gfa)ub) = (b)u({(σ, GFa)} {(Σ, (GFa)Ub)}) = {(Σ b, tt), (Σ, (GFa ((GFa)Ub))}

26 (LTL2BA) Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Optimization of VWAA If O 1 O 2 then replace the label a 2 in t 2 by a 2 a 1. If O 1 = O 2, replace both transitions by the transition (q, a 1 a 2, O 1 ). Figure: VWAA after apply generalized optimization rule.

27 (LTL2BA) Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Definition 12: (Progress formula). Let M be the minimal set containing all VWAA states of the form ψrp and all subformula of their right operands p. The VWAA states outside M, called progress formula.

28 (LTL2BA) Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Let A ϕ = (Q, Σ, δ, I, F ) be a VWAA. Define G A = (Q, Σ, δ, I, T ) - δ (O) = n δ O (q i ), where i=1 {(Σ, {q i })}if O contains a progress non-alternating formula and q i is an alternating formula, δ O (q i ) = or O contains a progress formula and q is an alternating non-progress formula δ(q i ) otherwise - T = {T f f F } where T f = {(O, α, O ) f / O or ( β, O ) δ(f ), (γ, O ) f O f δ(f ) such that f / O, α = β γ, and O = O O )}.

29 (LTL2BA) Example Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Let ψ = GFa Fb tt:{3} a:{2, 3} b:{2, 3} start {1, 2} {1} Figure: A VWAA A ψ tt:{2} Figure: A TGBA G ψ corresponding to the VWAA of Figure 3.

30 (LTL2BA) Example Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA Find δ (GF a F b ) - We have F b is progress formula and non-alternating, GF a is an alternating formula. - δ (GF a F b ) = δ(gf a ) δ(f b ) - In LTL2BA: δ(gf a ) = {(Σ, GF a )} - In LTL3BA: δ(gf a ) = {(Σ a, GF a ), (Σ, GF a F b )} δ (GF a F b ) = {(Σ b, GF a ), (Σ, GF a F b )} - (GF a F b, Σ b, GF a ) T Fb, T Fa - (GF a F b, Σ, GF a F b ) T Fa

31 (LTL2BA) Optimization of BA Alternating Formula Improvements in LTL to VWAA Translation Improvements in VWAA to TGBA Translation Optimization of BA New rule states q 1 and q 2 can be merged if δ(q 1 )[q 1 /r] = δ(q 2 )[q 2 /r], where r is a fresh artificial state and δ(q)[q/r] is a δ(q) with all occurrences of q as a target node replaced by r.

32 (LTL2BA) - The translation proceeds in three basic steps: LTL formula is translated into a very weak alternating automaton (VWAA) VWAA is then translated into a transition-based generalized Büchi automaton (TGBA) TGBA is transformed into Büchi automaton (BA) - Each of the three automata is simplified during the translation - LTL2BA implementation is available at following address: - PAT is using LTL2BA, replace LTL2BA by LTL3BA

33 (LTL2BA) References Paul Gastin and Denis Oddoux, Fast LTL to Büchi Automata Translation, Tom Babiak, Mojmr Ketnsk, Vojtch ehk, Jan Strejek, LTL to Büchi Automata Translation: Fast and More Deterministic*, Kousha Etessami and Gerard J.Holzmann, Optimizing Büchi automata, O.Kupferman and M.Vardi, Weak alternating automata are not that weak, 1997.

Büchi Automata and Linear Temporal Logic

Büchi Automata and Linear Temporal Logic Büchi Automata and Linear Temporal Logic Joshua D. Guttman Worcester Polytechnic Institute 18 February 2010 Guttman ( WPI ) Büchi & LTL 18 Feb 10 1 / 10 Büchi Automata Definition A Büchi automaton is a

More information

Minimising Deterministic Büchi Automata Precisely using SAT Solving

Minimising Deterministic Büchi Automata Precisely using SAT Solving Minimising Deterministic Büchi Automata Precisely using SAT Solving Rüdiger Ehlers Saarland University, Reactive Systems Group SAT 2010 July 14, 2010 Rüdiger Ehlers (SB) DBA Minimization SAT 2010 July

More information

Automata on Infinite words and LTL Model Checking

Automata on Infinite words and LTL Model Checking Automata on Infinite words and LTL Model Checking Rodica Condurache Lecture 4 Lecture 4 Automata on Infinite words and LTL Model Checking 1 / 35 Labeled Transition Systems Let AP be the (finite) set of

More information

Deterministic ω-automata for LTL: A safraless, compositional, and mechanically verified construction

Deterministic ω-automata for LTL: A safraless, compositional, and mechanically verified construction Deterministic ω-automata for LTL: A safraless, compositional, and mechanically verified construction Javier Esparza 1 Jan Křetínský 2 Salomon Sickert 1 1 Fakultät für Informatik, Technische Universität

More information

Effective Translation of LTL to Deterministic Rabin Automata: Beyond the (F,G)-Fragment

Effective Translation of LTL to Deterministic Rabin Automata: Beyond the (F,G)-Fragment Effective Translation of LTL to Deterministic Rabin Automata: Beyond the (F,G)-Fragment Tomáš Babiak, František Blahoudek, Mojmír Křetínský, and Jan Strejček Faculty of Informatics, Masaryk University,

More information

Almost Linear Büchi Automata

Almost Linear Büchi Automata Almost Linear Büchi Automata Tomáš Babiak Vojtěch Řehák Jan Strejček Faculty of Informatics Masaryk University Brno, Czech Republic {xbabiak, rehak, strejcek}@fi.muni.cz We introduce a new fragment of

More information

On the Relationship between LTL Normal Forms and Büchi Automata

On the Relationship between LTL Normal Forms and Büchi Automata On the Relationship between LTL Normal Forms and Büchi Automata Jianwen Li 1, Geguang Pu 1, Lijun Zhang 2, Zheng Wang 1, Jifeng He 1, and Kim G. Larsen 3 1 Software Engineering Institute East China Normal

More information

Automata-Theoretic Verification

Automata-Theoretic Verification Automata-Theoretic Verification Javier Esparza TU München Orna Kupferman The Hebrew University Moshe Y. Vardi Rice University 1 Introduction This chapter describes the automata-theoretic approach to the

More information

From Liveness to Promptness

From Liveness to Promptness From Liveness to Promptness Orna Kupferman Hebrew University Nir Piterman EPFL Moshe Y. Vardi Rice University Abstract Liveness temporal properties state that something good eventually happens, e.g., every

More information

Limit-Deterministic Büchi Automata for Linear Temporal Logic

Limit-Deterministic Büchi Automata for Linear Temporal Logic Limit-Deterministic Büchi Automata for Linear Temporal Logic Salomon Sickert, Javier Esparza, Stefan Jaax, and Jan Křetínský Technische Universität München Abstract. Limit-deterministic Büchi automata

More information

Temporal Logic. M φ. Outline. Why not standard logic? What is temporal logic? LTL CTL* CTL Fairness. Ralf Huuck. Kripke Structure

Temporal Logic. M φ. Outline. Why not standard logic? What is temporal logic? LTL CTL* CTL Fairness. Ralf Huuck. Kripke Structure Outline Temporal Logic Ralf Huuck Why not standard logic? What is temporal logic? LTL CTL* CTL Fairness Model Checking Problem model, program? M φ satisfies, Implements, refines property, specification

More information

Model Checking of Safety Properties

Model Checking of Safety Properties Model Checking of Safety Properties Orna Kupferman Hebrew University Moshe Y. Vardi Rice University October 15, 2010 Abstract Of special interest in formal verification are safety properties, which assert

More information

Temporal Logic. Stavros Tripakis University of California, Berkeley. We have designed a system. We want to check that it is correct.

Temporal Logic. Stavros Tripakis University of California, Berkeley. We have designed a system. We want to check that it is correct. EE 244: Fundamental Algorithms for System Modeling, Analysis, and Optimization Fall 2016 Temporal logic Stavros Tripakis University of California, Berkeley Stavros Tripakis (UC Berkeley) EE 244, Fall 2016

More information

970 JOURNAL OF SOFTWARE, VOL. 9, NO. 4, APRIL Conversion Algorithm of Linear-Time Temporal Logic to Büchi Automata

970 JOURNAL OF SOFTWARE, VOL. 9, NO. 4, APRIL Conversion Algorithm of Linear-Time Temporal Logic to Büchi Automata 970 JOURNAL OF SOFTWARE, VOL. 9, NO. 4, APRIL 2014 Conversion Algorithm of Linear-Time Temporal Logic to Büchi Automata Laixiang Shan a,c, Zheng Qin b,c, Shengnan Li a,c, Renwei Zhang b, Xiao Yang b a

More information

An On-the-fly Tableau Construction for a Real-Time Temporal Logic

An On-the-fly Tableau Construction for a Real-Time Temporal Logic #! & F $ F ' F " F % An On-the-fly Tableau Construction for a Real-Time Temporal Logic Marc Geilen and Dennis Dams Faculty of Electrical Engineering, Eindhoven University of Technology P.O.Box 513, 5600

More information

CS256/Spring 2008 Lecture #11 Zohar Manna. Beyond Temporal Logics

CS256/Spring 2008 Lecture #11 Zohar Manna. Beyond Temporal Logics CS256/Spring 2008 Lecture #11 Zohar Manna Beyond Temporal Logics Temporal logic expresses properties of infinite sequences of states, but there are interesting properties that cannot be expressed, e.g.,

More information

A Hierarchy for Accellera s Property Specification Language

A Hierarchy for Accellera s Property Specification Language A Hierarchy for Accellera s Property Specification Language Thomas Türk May 1st, 2005 Diploma Thesis University of Kaiserslautern Supervisor: Prof. Dr. Klaus Schneider Vorliegende Diplomarbeit wurde von

More information

Automata and Reactive Systems

Automata and Reactive Systems Automata and Reactive Systems Lecture WS 2002/2003 Prof. Dr. W. Thomas RWTH Aachen Preliminary version (Last change March 20, 2003) Translated and revised by S. N. Cho and S. Wöhrle German version by M.

More information

Tecniche di Specifica e di Verifica. Automata-based LTL Model-Checking

Tecniche di Specifica e di Verifica. Automata-based LTL Model-Checking Tecniche di Specifica e di Verifica Automata-based LTL Model-Checking Finite state automata A finite state automaton is a tuple A = (Σ,S,S 0,R,F) Σ: set of input symbols S: set of states -- S 0 : set of

More information

Verifying the LTL to Büchi Automata Translation via Very Weak Alternating Automata

Verifying the LTL to Büchi Automata Translation via Very Weak Alternating Automata Verifying the LTL to Büchi Automata Translation via Very Weak Alternating Automata Simon Jantsch 1(B) and Michael Norrish 2 1 TU Dresden, Dresden, Germany simon.jantsch@gmail.com 2 Data61, CSIRO and Australian

More information

Introduction. Büchi Automata and Model Checking. Outline. Büchi Automata. The simplest computation model for infinite behaviors is the

Introduction. Büchi Automata and Model Checking. Outline. Büchi Automata. The simplest computation model for infinite behaviors is the Introduction Büchi Automata and Model Checking Yih-Kuen Tsay Department of Information Management National Taiwan University FLOLAC 2009 The simplest computation model for finite behaviors is the finite

More information

Temporal logics and explicit-state model checking. Pierre Wolper Université de Liège

Temporal logics and explicit-state model checking. Pierre Wolper Université de Liège Temporal logics and explicit-state model checking Pierre Wolper Université de Liège 1 Topics to be covered Introducing explicit-state model checking Finite automata on infinite words Temporal Logics and

More information

Automata Construction for PSL

Automata Construction for PSL Automata Construction for Doron Bustan 1 Dana Fisman 2 John Havlicek 1 dbustan@freescale.com dana.fisman@weizmann.ac.il john.havlicek@freescale.com 1 Freescale Semiconductor, Inc. 2 Weizmann Institute

More information

LTL with Arithmetic and its Applications in Reasoning about Hierarchical Systems

LTL with Arithmetic and its Applications in Reasoning about Hierarchical Systems This space is reserved for the EPiC Series header, do not use it LTL with Arithmetic and its Applications in Reasoning about Hierarchical Systems Rachel Faran and Orna Kupferman The Hebrew University,

More information

Alan Bundy. Automated Reasoning LTL Model Checking

Alan Bundy. Automated Reasoning LTL Model Checking Automated Reasoning LTL Model Checking Alan Bundy Lecture 9, page 1 Introduction So far we have looked at theorem proving Powerful, especially where good sets of rewrite rules or decision procedures have

More information

Computer-Aided Program Design

Computer-Aided Program Design Computer-Aided Program Design Spring 2015, Rice University Unit 3 Swarat Chaudhuri February 5, 2015 Temporal logic Propositional logic is a good language for describing properties of program states. However,

More information

Efficient Model Checking of Safety Properties

Efficient Model Checking of Safety Properties Efficient Model Checking of Safety Properties Timo Latvala timo.latvala@hut.fi Laboratory for Theoretical Computer Science Helsinki University of Technology Finland Spin 2003 p.1/16 Introduction Safety

More information

Languages, logics and automata

Languages, logics and automata Languages, logics and automata Anca Muscholl LaBRI, Bordeaux, France EWM summer school, Leiden 2011 1 / 89 Before all that.. Sonia Kowalewskaya Emmy Noether Julia Robinson All this attention has been gratifying

More information

a Hebrew University b Weizmann Institute c Rice University

a Hebrew University b Weizmann Institute c Rice University Once and For All Orna Kupferman a, Amir Pnueli b,1, Moshe Y. Vardi c a Hebrew University b Weizmann Institute c Rice University Abstract It has long been known that past-time operators add no expressive

More information

Büchi Automata and Their Determinization

Büchi Automata and Their Determinization Büchi Automata and Their Determinization Edinburgh, October 215 Plan of the Day 1. Büchi automata and their determinization 2. Infinite games 3. Rabin s Tree Theorem 4. Decidability of monadic theories

More information

Linear Temporal Logic and Büchi Automata

Linear Temporal Logic and Büchi Automata Linear Temporal Logic and Büchi Automata Yih-Kuen Tsay Department of Information Management National Taiwan University FLOLAC 2009 Yih-Kuen Tsay (SVVRL @ IM.NTU) Linear Temporal Logic and Büchi Automata

More information

Logic Model Checking

Logic Model Checking Logic Model Checking Lecture Notes 10:18 Caltech 101b.2 January-March 2004 Course Text: The Spin Model Checker: Primer and Reference Manual Addison-Wesley 2003, ISBN 0-321-22862-6, 608 pgs. the assignment

More information

Tecniche di Specifica e di Verifica. Automata-based LTL Model-Checking

Tecniche di Specifica e di Verifica. Automata-based LTL Model-Checking Tecniche di Specifica e di Verifica Automata-based LTL Model-Checking Finite state automata A finite state automaton is a tuple A = (S,S,S 0,R,F) S: set of input symbols S: set of states -- S 0 : set of

More information

Push-down Automata = FA + Stack

Push-down Automata = FA + Stack Push-down Automata = FA + Stack PDA Definition A push-down automaton M is a tuple M = (Q,, Γ, δ, q0, F) where Q is a finite set of states is the input alphabet (of terminal symbols, terminals) Γ is the

More information

From Liveness to Promptness

From Liveness to Promptness From Liveness to Promptness Orna Kupferman 1, Nir Piterman 2, and Moshe Y. Vardi 3 1 Hebrew University 2 Ecole Polytechnique Fédéral de Lausanne (EPFL) 3 Rice University Abstract. Liveness temporal properties

More information

Classes and conversions

Classes and conversions Classes and conversions Regular expressions Syntax: r = ε a r r r + r r Semantics: The language L r of a regular expression r is inductively defined as follows: L =, L ε = {ε}, L a = a L r r = L r L r

More information

Lecture Notes on Emptiness Checking, LTL Büchi Automata

Lecture Notes on Emptiness Checking, LTL Büchi Automata 15-414: Bug Catching: Automated Program Verification Lecture Notes on Emptiness Checking, LTL Büchi Automata Matt Fredrikson André Platzer Carnegie Mellon University Lecture 18 1 Introduction We ve seen

More information

Lattice Automata. Orna Kupferman and Yoad Lustig

Lattice Automata. Orna Kupferman and Yoad Lustig Lattice Automata Orna Kupferman and Yoad Lustig Hebrew University, School of Engineering and Computer Science, Jerusalem 91904, Israel Email: {orna,yoadl}@cs.huji.ac.il Abstract. Several verification methods

More information

Designing Petri Net Supervisors from LTL Specifications

Designing Petri Net Supervisors from LTL Specifications Robotics: Science and Systems 20 Los Angeles, CA, USA, June 27-30, 20 Designing Petri Net Supervisors from LTL Specifications Bruno Lacerda and Pedro U. Lima Institute for Systems and Robotics Instituto

More information

arxiv: v1 [cs.lo] 17 Jun 2014

arxiv: v1 [cs.lo] 17 Jun 2014 On MITL and alternating timed automata over infinite words Thomas Brihaye 1, Morgane Estiévenart 1, and Gilles Geeraerts 2 1 UMons, Belgium, 2 U.L.B., Belgium arxiv:1406.4395v1 [cs.lo] 17 Jun 2014 Abstract.

More information

Representing Arithmetic Constraints with Finite Automata: An Overview

Representing Arithmetic Constraints with Finite Automata: An Overview Representing Arithmetic Constraints with Finite Automata: An Overview Bernard Boigelot Pierre Wolper Université de Liège Motivation Linear numerical constraints are a very common and useful formalism (our

More information

On the Succinctness of Nondeterminizm

On the Succinctness of Nondeterminizm On the Succinctness of Nondeterminizm Benjamin Aminof and Orna Kupferman Hebrew University, School of Engineering and Computer Science, Jerusalem 91904, Israel Email: {benj,orna}@cs.huji.ac.il Abstract.

More information

Failure Diagnosis of Discrete Event Systems With Linear-Time Temporal Logic Specifications

Failure Diagnosis of Discrete Event Systems With Linear-Time Temporal Logic Specifications Failure Diagnosis of Discrete Event Systems With Linear-Time Temporal Logic Specifications Shengbing Jiang and Ratnesh Kumar Abstract The paper studies failure diagnosis of discrete event systems with

More information

Automata-based Verification - III

Automata-based Verification - III COMP30172: Advanced Algorithms Automata-based Verification - III Howard Barringer Room KB2.20: email: howard.barringer@manchester.ac.uk March 2009 Third Topic Infinite Word Automata Motivation Büchi Automata

More information

Tableau-Based Automata Construction for Dynamic Linear Time Temporal Logic

Tableau-Based Automata Construction for Dynamic Linear Time Temporal Logic Tableau-Based Automata Construction for Dynamic Linear Time Temporal Logic Laura Giordano Università del Piemonte Orientale Alessandria, Italy laura@mfn.unipmn.it Alberto Martelli Università di Torino

More information

Helsinki University of Technology Laboratory for Theoretical Computer Science Research Reports 66

Helsinki University of Technology Laboratory for Theoretical Computer Science Research Reports 66 Helsinki University of Technology Laboratory for Theoretical Computer Science Research Reports 66 Teknillisen korkeakoulun tietojenkäsittelyteorian laboratorion tutkimusraportti 66 Espoo 2000 HUT-TCS-A66

More information

Theory of Computation

Theory of Computation Thomas Zeugmann Hokkaido University Laboratory for Algorithmics http://www-alg.ist.hokudai.ac.jp/ thomas/toc/ Lecture 3: Finite State Automata Motivation In the previous lecture we learned how to formalize

More information

Stéphane Demri Arnaud Sangnier. When Model-Checking Freeze LTL over Counter Machines Becomes Decidable. Research Report LSV-10-05

Stéphane Demri Arnaud Sangnier. When Model-Checking Freeze LTL over Counter Machines Becomes Decidable. Research Report LSV-10-05 Stéphane Demri Arnaud Sangnier When Model-Checking Freeze LTL over Counter Machines Becomes Decidable Research Report LSV-10-05 February 2010 When Model-Checking Freeze LTL over Counter Machines Becomes

More information

Weak Alternating Automata Are Not That Weak

Weak Alternating Automata Are Not That Weak Weak Alternating Automata Are Not That Weak Orna Kupferman Hebrew University Moshe Y. Vardi Rice University Abstract Automata on infinite words are used for specification and verification of nonterminating

More information

Rabin Theory and Game Automata An Introduction

Rabin Theory and Game Automata An Introduction Rabin Theory and Game Automata An Introduction Ting Zhang Stanford University November 2002 Logic Seminar 1 Outline 1. Monadic second-order theory of two successors (S2S) 2. Rabin Automata 3. Game Automata

More information

Chapter 3: Linear temporal logic

Chapter 3: Linear temporal logic INFOF412 Formal verification of computer systems Chapter 3: Linear temporal logic Mickael Randour Formal Methods and Verification group Computer Science Department, ULB March 2017 1 LTL: a specification

More information

Homework 2: Temporal logic

Homework 2: Temporal logic ICS-E5010 Computer-Aided Verification and Synthesis, Spring 2016 Stavros Tripakis Homework 2: Temporal logic Assigned: January 20, 2016 Due: February 1, 2016 Total: 235 points. 1. (20 points) Two formulae

More information

Logic and Automata I. Wolfgang Thomas. EATCS School, Telc, July 2014

Logic and Automata I. Wolfgang Thomas. EATCS School, Telc, July 2014 Logic and Automata I EATCS School, Telc, July 2014 The Plan We present automata theory as a tool to make logic effective. Four parts: 1. Some history 2. Automata on infinite words First step: MSO-logic

More information

Simple and Efficient Translation from LTL Formulas to Büchi Automata

Simple and Efficient Translation from LTL Formulas to Büchi Automata Electronic Notes in Theoretical Computer Science 66 No. 2 (2002) URL: http://www.elsevier.nl/locate/entcs/volume66.html 15 pages Simple and Efficient Translation from LTL Formulas to Büchi Automata Xavier

More information

Minimization of Tree Automata

Minimization of Tree Automata Universität des Saarlandes Naturwissenschaftlich-Technische Fakultät 1 Fachrichtung Informatik Bachelor-Studiengang Informatik Bachelor s Thesis Minimization of Tree Automata submitted by Thomas von Bomhard

More information

Visibly Linear Dynamic Logic

Visibly Linear Dynamic Logic Visibly Linear Dynamic Logic Joint work with Alexander Weinert (Saarland University) Martin Zimmermann Saarland University September 8th, 2016 Highlights Conference, Brussels, Belgium Martin Zimmermann

More information

Java II Finite Automata I

Java II Finite Automata I Java II Finite Automata I Bernd Kiefer Bernd.Kiefer@dfki.de Deutsches Forschungszentrum für künstliche Intelligenz November, 23 Processing Regular Expressions We already learned about Java s regular expression

More information

A Tight Lower Bound for Determinization of Transition Labeled Büchi Automata

A Tight Lower Bound for Determinization of Transition Labeled Büchi Automata A Tight Lower Bound for Determinization of Transition Labeled Büchi Automata Thomas Colcombet, Konrad Zdanowski CNRS JAF28, Fontainebleau June 18, 2009 Finite Automata A finite automaton is a tuple A =

More information

Synthesis of Distributed Control and Communication Schemes from Global LTL Specifications

Synthesis of Distributed Control and Communication Schemes from Global LTL Specifications Synthesis of Distributed Control and Communication Schemes from Global LTL Specifications Yushan Chen, Xu Chu Ding, and Calin Belta Abstract We introduce a technique for synthesis of control and communication

More information

Automata and Formal Languages - CM0081 Non-Deterministic Finite Automata

Automata and Formal Languages - CM0081 Non-Deterministic Finite Automata Automata and Formal Languages - CM81 Non-Deterministic Finite Automata Andrés Sicard-Ramírez Universidad EAFIT Semester 217-2 Non-Deterministic Finite Automata (NFA) Introduction q i a a q j a q k The

More information

Temporal Logic with Past is Exponentially More Succinct

Temporal Logic with Past is Exponentially More Succinct Temporal Logic with Past is Exponentially More Succinct Nicolas Markey Lab. Informatique Fondamentale d Orléans Univ. Orléans & CNRS FRE 2490 Rue Léonard de Vinci - BP 6759 45067 Orléans Cedex 2 - France

More information

September 11, Second Part of Regular Expressions Equivalence with Finite Aut

September 11, Second Part of Regular Expressions Equivalence with Finite Aut Second Part of Regular Expressions Equivalence with Finite Automata September 11, 2013 Lemma 1.60 If a language is regular then it is specified by a regular expression Proof idea: For a given regular language

More information

Comparison of LTL to Deterministic Rabin Automata Translators

Comparison of LTL to Deterministic Rabin Automata Translators Comparison of LTL to Deterministic Rabin Automata Translators František Blahoudek, Mojmír Křetínský, and Jan Strejček Faculty of Informatics, Masaryk University, Brno, Czech Republic {xblahoud, kretinsky,

More information

Automata-based Verification - III

Automata-based Verification - III CS3172: Advanced Algorithms Automata-based Verification - III Howard Barringer Room KB2.20/22: email: howard.barringer@manchester.ac.uk March 2005 Third Topic Infinite Word Automata Motivation Büchi Automata

More information

FORMAL LANGUAGES, AUTOMATA AND COMPUTABILITY

FORMAL LANGUAGES, AUTOMATA AND COMPUTABILITY 15-453 FORMAL LANGUAGES, AUTOMATA AND COMPUTABILITY REVIEW for MIDTERM 1 THURSDAY Feb 6 Midterm 1 will cover everything we have seen so far The PROBLEMS will be from Sipser, Chapters 1, 2, 3 It will be

More information

CHURCH SYNTHESIS PROBLEM and GAMES

CHURCH SYNTHESIS PROBLEM and GAMES p. 1/? CHURCH SYNTHESIS PROBLEM and GAMES Alexander Rabinovich Tel-Aviv University, Israel http://www.tau.ac.il/ rabinoa p. 2/? Plan of the Course 1. The Church problem - logic and automata. 2. Games -

More information

The theory of regular cost functions.

The theory of regular cost functions. The theory of regular cost functions. Denis Kuperberg PhD under supervision of Thomas Colcombet Hebrew University of Jerusalem ERC Workshop on Quantitative Formal Methods Jerusalem, 10-05-2013 1 / 30 Introduction

More information

Optimal Translation of LTL to Limit Deterministic Automata

Optimal Translation of LTL to Limit Deterministic Automata Optimal Translation of LTL to Limit Deterministic Automata Dileep Kini and Mahesh Viswanathan University of Illinois at Urbana-Champaign, Department of Computer Science Abstract. A crucial step in model

More information

Decision Procedures for CTL

Decision Procedures for CTL Decision Procedures for CTL Oliver Friedmann and Markus Latte Dept. of Computer Science, University of Munich, Germany Abstract. We give an overview over three serious attempts to devise an effective decision

More information

Note on winning positions on pushdown games with omega-regular winning conditions

Note on winning positions on pushdown games with omega-regular winning conditions Note on winning positions on pushdown games with omega-regular winning conditions Olivier Serre To cite this version: Olivier Serre. Note on winning positions on pushdown games with omega-regular winning

More information

Büchi Automata and their closure properties. - Ajith S and Ankit Kumar

Büchi Automata and their closure properties. - Ajith S and Ankit Kumar Büchi Automata and their closure properties - Ajith S and Ankit Kumar Motivation Conventional programs accept input, compute, output result, then terminate Reactive program : not expected to terminate

More information

2. Elements of the Theory of Computation, Lewis and Papadimitrou,

2. Elements of the Theory of Computation, Lewis and Papadimitrou, Introduction Finite Automata DFA, regular languages Nondeterminism, NFA, subset construction Regular Epressions Synta, Semantics Relationship to regular languages Properties of regular languages Pumping

More information

(b) If G=({S}, {a}, {S SS}, S) find the language generated by G. [8+8] 2. Convert the following grammar to Greibach Normal Form G = ({A1, A2, A3},

(b) If G=({S}, {a}, {S SS}, S) find the language generated by G. [8+8] 2. Convert the following grammar to Greibach Normal Form G = ({A1, A2, A3}, Code No: 07A50501 R07 Set No. 2 III B.Tech I Semester Examinations,MAY 2011 FORMAL LANGUAGES AND AUTOMATA THEORY Computer Science And Engineering Time: 3 hours Max Marks: 80 Answer any FIVE Questions All

More information

Cooperative Decentralized Multi-agent Control under Local LTL Tasks and Connectivity Constraints

Cooperative Decentralized Multi-agent Control under Local LTL Tasks and Connectivity Constraints Cooperative Decentralized Multi-agent Control under Local LTL Tasks and Connectivity Constraints Meng Guo, Jana Tumova and Dimos V. Dimarogonas Abstract We propose a framework for the decentralized control

More information

What we have done so far

What we have done so far What we have done so far DFAs and regular languages NFAs and their equivalence to DFAs Regular expressions. Regular expressions capture exactly regular languages: Construct a NFA from a regular expression.

More information

Alternation Removal in Büchi Automata

Alternation Removal in Büchi Automata Alternation Removal in Büchi Automata Udi Boker, Orna Kupferman and Adin Rosenberg School of Computer Science and Engineering, Hebrew University, Israel. Abstract. Alternating automata play a key role

More information

Sri vidya college of engineering and technology

Sri vidya college of engineering and technology Unit I FINITE AUTOMATA 1. Define hypothesis. The formal proof can be using deductive proof and inductive proof. The deductive proof consists of sequence of statements given with logical reasoning in order

More information

Chapter 3. Regular grammars

Chapter 3. Regular grammars Chapter 3 Regular grammars 59 3.1 Introduction Other view of the concept of language: not the formalization of the notion of effective procedure, but set of words satisfying a given set of rules Origin

More information

LTL is Closed Under Topological Closure

LTL is Closed Under Topological Closure LTL is Closed Under Topological Closure Grgur Petric Maretić, Mohammad Torabi Dashti, David Basin Department of Computer Science, ETH Universitätstrasse 6 Zürich, Switzerland Abstract We constructively

More information

Taming Past LTL and Flat Counter Systems

Taming Past LTL and Flat Counter Systems Taming Past LTL and Flat Counter Systems Amit Kumar Dhar LIAFA, Univ Paris Diderot, Paris Cité Sorbonne, CNRS, France April 2, 2012 Joint work with : Stéphane Demri(LSV) and Arnaud Sangnier(LIAFA) LIAFA

More information

SATISFIABILITY GAMES FOR BRANCHING-TIME LOGICS

SATISFIABILITY GAMES FOR BRANCHING-TIME LOGICS Logical Methods in Computer Science Vol. 9(4:5)2013, pp. 1 36 www.lmcs-online.org Submitted Feb. 5, 2013 Published Oct. 16, 2013 SATISFIABILITY GAMES FOR BRANCHING-TIME LOGICS OLIVER FRIEDMANN a, MARKUS

More information

Decision Procedures for CTL

Decision Procedures for CTL Decision Procedures for CTL Oliver Friedmann 1 Markus Latte 1 1 Dept. of Computer Science, Ludwig-Maximilians-University, Munich, Germany CLoDeM Edinburgh, 15 July 2010 Introduction to CTL Origin: Emerson

More information

Theory of Computation (IV) Yijia Chen Fudan University

Theory of Computation (IV) Yijia Chen Fudan University Theory of Computation (IV) Yijia Chen Fudan University Review language regular context-free machine DFA/ NFA PDA syntax regular expression context-free grammar Pushdown automata Definition A pushdown automaton

More information

Automata Theory for Presburger Arithmetic Logic

Automata Theory for Presburger Arithmetic Logic Automata Theory for Presburger Arithmetic Logic References from Introduction to Automata Theory, Languages & Computation and Constraints in Computational Logic Theory & Application Presented by Masood

More information

ω-automata Automata that accept (or reject) words of infinite length. Languages of infinite words appear:

ω-automata Automata that accept (or reject) words of infinite length. Languages of infinite words appear: ω-automata ω-automata Automata that accept (or reject) words of infinite length. Languages of infinite words appear: in verification, as encodings of non-terminating executions of a program. in arithmetic,

More information

Logic in Automatic Verification

Logic in Automatic Verification Logic in Automatic Verification Javier Esparza Sofware Reliability and Security Group Institute for Formal Methods in Computer Science University of Stuttgart Many thanks to Abdelwaheb Ayari, David Basin,

More information

Efficient Model Checking of Safety Properties

Efficient Model Checking of Safety Properties Efficient Model Checking of Safety Properties Timo Latvala Laboratory for Theoretical Computer Science Helsinki University of Technology P.O. Box 9205 FIN-02015 HUT Finland Timo.Latvala@hut.fi Abstract.

More information

FINITE MEMORY DETERMINACY

FINITE MEMORY DETERMINACY p. 1/? FINITE MEMORY DETERMINACY Alexander Rabinovich Department of Computer Science Tel-Aviv University p. 2/? Plan 1. Finite Memory Strategies. 2. Finite Memory Determinacy of Muller games. 3. Latest

More information

Helsinki University of Technology Laboratory for Theoretical Computer Science Research Reports 83

Helsinki University of Technology Laboratory for Theoretical Computer Science Research Reports 83 Helsinki University of Technology Laboratory for Theoretical Computer Science Research Reports 83 Teknillisen korkeakoulun tietojenkäsittelyteorian laboratorion tutkimusraportti 83 Espoo 2003 HUT-TCS-A83

More information

CMSC 330: Organization of Programming Languages. Theory of Regular Expressions Finite Automata

CMSC 330: Organization of Programming Languages. Theory of Regular Expressions Finite Automata : Organization of Programming Languages Theory of Regular Expressions Finite Automata Previous Course Review {s s defined} means the set of string s such that s is chosen or defined as given s A means

More information

Chapter 5: Linear Temporal Logic

Chapter 5: Linear Temporal Logic Chapter 5: Linear Temporal Logic Prof. Ali Movaghar Verification of Reactive Systems Spring 91 Outline We introduce linear temporal logic (LTL), a logical formalism that is suited for specifying LT properties.

More information

Timo Latvala. March 7, 2004

Timo Latvala. March 7, 2004 Reactive Systems: Safety, Liveness, and Fairness Timo Latvala March 7, 2004 Reactive Systems: Safety, Liveness, and Fairness 14-1 Safety Safety properties are a very useful subclass of specifications.

More information

Chapter Five: Nondeterministic Finite Automata

Chapter Five: Nondeterministic Finite Automata Chapter Five: Nondeterministic Finite Automata From DFA to NFA A DFA has exactly one transition from every state on every symbol in the alphabet. By relaxing this requirement we get a related but more

More information

C6.2 Push-Down Automata

C6.2 Push-Down Automata Theory of Computer Science April 5, 2017 C6. Context-free Languages: Push-down Automata Theory of Computer Science C6. Context-free Languages: Push-down Automata Malte Helmert University of Basel April

More information

Model Checking LTL with Regular Valuations for Pushdown Systems 1

Model Checking LTL with Regular Valuations for Pushdown Systems 1 Model Checking LTL with Regular Valuations for Pushdown Systems 1 Javier Esparza Division of Informatics University of Edinburgh Edinburgh EH9 3JZ United Kingdom E-mail: jav@dcs.ed.ac.uk and Antonín Kučera

More information

Chapter 5: Linear Temporal Logic

Chapter 5: Linear Temporal Logic Chapter 5: Linear Temporal Logic Prof. Ali Movaghar Verification of Reactive Systems Spring 94 Outline We introduce linear temporal logic (LTL), a logical formalism that is suited for specifying LT properties.

More information

CDS 270 (Fall 09) - Lecture Notes for Assignment 8.

CDS 270 (Fall 09) - Lecture Notes for Assignment 8. CDS 270 (Fall 09) - Lecture Notes for Assignment 8. ecause this part of the course has no slides or textbook, we will provide lecture supplements that include, hopefully, enough discussion to complete

More information

On Regular Temporal Logics with Past

On Regular Temporal Logics with Past , On Regular Temporal Logics with Past Christian Dax 1, Felix Klaedtke 1, and Martin Lange 2 1 ETH Zurich, Switzerland 2 Ludwig-Maximilians-University Munich, Germany Abstract. The IEEE standardized Property

More information

Computational Models Lecture 2 1

Computational Models Lecture 2 1 Computational Models Lecture 2 1 Handout Mode Iftach Haitner. Tel Aviv University. October 30, 2017 1 Based on frames by Benny Chor, Tel Aviv University, modifying frames by Maurice Herlihy, Brown University.

More information

Focus Games for Satisfiability and Completeness of Temporal Logic

Focus Games for Satisfiability and Completeness of Temporal Logic Focus Games for Satisfiability and Completeness of Temporal Logic Martin Lange Colin Stirling LFCS, Division of Informatics, University of Edinburgh, JCMB, King s Buildings, Edinburgh, EH9 3JZ {martin,cps}@dcs.ed.ac.uk

More information