src/HOLCF/IOA/ABP/Impl.thy
changeset 25131 2c8caac48ade
parent 19738 1ac610922636
child 35174 e15040ae75d7
--- a/src/HOLCF/IOA/ABP/Impl.thy	Sun Oct 21 14:21:45 2007 +0200
+++ b/src/HOLCF/IOA/ABP/Impl.thy	Sun Oct 21 14:21:48 2007 +0200
@@ -13,21 +13,24 @@
   'm impl_state = "'m sender_state * 'm receiver_state * 'm packet list * bool list"
   (*  sender_state   *  receiver_state   *    srch_state  * rsch_state *)
 
-constdefs
+definition
+ impl_ioa :: "('m action, 'm impl_state)ioa" where
+ "impl_ioa = (sender_ioa || receiver_ioa || srch_ioa || rsch_ioa)"
 
- impl_ioa    :: "('m action, 'm impl_state)ioa"
- "impl_ioa == (sender_ioa || receiver_ioa || srch_ioa || rsch_ioa)"
-
- sen         :: "'m impl_state => 'm sender_state"
- "sen == fst"
+definition
+ sen :: "'m impl_state => 'm sender_state" where
+ "sen = fst"
 
- rec         :: "'m impl_state => 'm receiver_state"
- "rec == fst o snd"
+definition
+ rec :: "'m impl_state => 'm receiver_state" where
+ "rec = fst o snd"
 
- srch        :: "'m impl_state => 'm packet list"
- "srch == fst o snd o snd"
+definition
+ srch :: "'m impl_state => 'm packet list" where
+ "srch = fst o snd o snd"
 
- rsch        :: "'m impl_state => bool list"
- "rsch == snd o snd o snd"
+definition
+ rsch :: "'m impl_state => bool list" where
+ "rsch = snd o snd o snd"
 
 end