src/HOL/UNITY/WFair.thy
changeset 35416 d8d7d1b785af
parent 32693 6c6b1ba5e71e
child 35417 47ee18b6ae32
--- a/src/HOL/UNITY/WFair.thy	Wed Feb 24 11:55:52 2010 +0100
+++ b/src/HOL/UNITY/WFair.thy	Mon Mar 01 13:40:23 2010 +0100
@@ -1,5 +1,4 @@
 (*  Title:      HOL/UNITY/WFair
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
 
@@ -33,16 +32,17 @@
 is the impossibility law for leads-to.
 *}
 
-constdefs
+definition
 
   --{*This definition specifies conditional fairness.  The rest of the theory
       is generic to all forms of fairness.  To get weak fairness, conjoin
       the inclusion below with @{term "A \<subseteq> Domain act"}, which specifies 
       that the action is enabled over all of @{term A}.*}
-  transient :: "'a set => 'a program set"
+  transient :: "'a set => 'a program set" where
     "transient A == {F. \<exists>act\<in>Acts F. act``A \<subseteq> -A}"
 
-  ensures :: "['a set, 'a set] => 'a program set"       (infixl "ensures" 60)
+definition
+  ensures :: "['a set, 'a set] => 'a program set"       (infixl "ensures" 60) where
     "A ensures B == (A-B co A \<union> B) \<inter> transient (A-B)"
 
 
@@ -59,13 +59,11 @@
   | Union:  "\<forall>A \<in> S. (A,B) \<in> leads F ==> (Union S, B) \<in> leads F"
 
 
-constdefs
-
-  leadsTo :: "['a set, 'a set] => 'a program set"    (infixl "leadsTo" 60)
+definition leadsTo :: "['a set, 'a set] => 'a program set" (infixl "leadsTo" 60) where
      --{*visible version of the LEADS-TO relation*}
     "A leadsTo B == {F. (A,B) \<in> leads F}"
   
-  wlt :: "['a program, 'a set] => 'a set"
+definition wlt :: "['a program, 'a set] => 'a set" where
      --{*predicate transformer: the largest set that leads to @{term B}*}
     "wlt F B == Union {A. F \<in> A leadsTo B}"
 
@@ -641,4 +639,4 @@
 apply blast+
 done
 
-end
+end
\ No newline at end of file