src/HOL/Modelcheck/CTL.thy
author wenzelm
Fri, 26 Oct 2001 23:58:21 +0200
changeset 11952 b10f1e8862f4
parent 7295 fe09a0c5cebe
child 17272 c63e5220ed77
permissions -rw-r--r--
* Pure: method 'atomize' presents local goal premises as object-level statements (atomic meta-level propositions); setup controlled via rewrite rules declarations of 'atomize' attribute; example application: 'induct' method with proper rule statements in improper proof *scripts*;

(*  Title:      HOL/Modelcheck/CTL.thy
    ID:         $Id$
    Author:     Olaf Mueller, Jan Philipps, Robert Sandner
    Copyright   1997  TU Muenchen
*)

CTL = MuCalculus + 


types
  'a trans  = "('a * 'a) set"

consts
  CEX   ::"['a trans,'a pred, 'a]=>bool"
  EG    ::"['a trans,'a pred]=> 'a pred"

defs
  CEX_def  "CEX N f u == (? v. (f v & (u,v):N))"
  EG_def   "EG N f == nu (% Q. % u.(f u & CEX N Q u))"

end