src/HOL/UNITY/Simple/Reach.thy
changeset 36866 426d5781bb25
parent 35416 d8d7d1b785af
child 37936 1e4c5015a72e
--- a/src/HOL/UNITY/Simple/Reach.thy	Wed May 12 15:25:58 2010 +0200
+++ b/src/HOL/UNITY/Simple/Reach.thy	Wed May 12 16:44:49 2010 +0200
@@ -17,20 +17,20 @@
 
   edges :: "(vertex*vertex) set"
 
-definition asgt :: "[vertex,vertex] => (state*state) set" where
-    "asgt u v == {(s,s'). s' = s(v:= s u | s v)}"
+definition asgt :: "[vertex,vertex] => (state*state) set"
+  where "asgt u v = {(s,s'). s' = s(v:= s u | s v)}"
 
-definition Rprg :: "state program" where
-    "Rprg == mk_total_program ({%v. v=init}, \<Union>(u,v)\<in>edges. {asgt u v}, UNIV)"
+definition Rprg :: "state program"
+  where "Rprg = mk_total_program ({%v. v=init}, \<Union>(u,v)\<in>edges. {asgt u v}, UNIV)"
 
-definition reach_invariant :: "state set" where
-    "reach_invariant == {s. (\<forall>v. s v --> (init, v) \<in> edges^*) & s init}"
+definition reach_invariant :: "state set"
+  where "reach_invariant = {s. (\<forall>v. s v --> (init, v) \<in> edges^*) & s init}"
 
-definition fixedpoint :: "state set" where
-    "fixedpoint == {s. \<forall>(u,v)\<in>edges. s u --> s v}"
+definition fixedpoint :: "state set"
+  where "fixedpoint = {s. \<forall>(u,v)\<in>edges. s u --> s v}"
 
-definition metric :: "state => nat" where
-    "metric s == card {v. ~ s v}"
+definition metric :: "state => nat"
+  where "metric s = card {v. ~ s v}"
 
 
 text{**We assume that the set of vertices is finite*}