src/ZF/UNITY/FP.thy
author paulson
Tue, 21 May 2002 13:06:36 +0200
changeset 13168 afcbca3498b0
parent 12195 ed2893765a08
child 14092 68da54626309
permissions -rw-r--r--
converted domrange to Isar and merged with equalities

(*  Title:      ZF/UNITY/FP.thy
    ID:         $Id$
    Author:     Sidi O Ehmety, Computer Laboratory
    Copyright   2001  University of Cambridge

Fixed Point of a Program

From Misra, "A Logic for Concurrent Programming", 1994

Theory ported from HOL.
*)

FP = UNITY +

constdefs   
  FP_Orig :: i=>i
    "FP_Orig(F) == Union({A:Pow(state). ALL B. F : stable(A Int B)})"

  FP :: i=>i
    "FP(F) == {s:state. F : stable({s})}"

end