src/HOL/Modelcheck/CTL.thy
author blanchet
Thu, 29 Apr 2010 01:17:14 +0200
changeset 36555 8ff45c2076da
parent 35416 d8d7d1b785af
permissions -rw-r--r--
expand combinators in Isar proofs constructed by Sledgehammer; this requires shuffling around a couple of functions previously defined in Refute

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

theory CTL
imports MuCalculus
begin

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

definition CEX :: "['a trans,'a pred, 'a]=>bool" where
  "CEX N f u == (? v. (f v & (u,v):N))"

definition EG ::"['a trans,'a pred]=> 'a pred" where
  "EG N f == nu (% Q. % u.(f u & CEX N Q u))"

end