src/HOLCF/IOA/meta_theory/Automata.thy
changeset 3275 3f53f2c876f4
parent 3071 981258186b71
child 3433 2de17c994071
--- a/src/HOLCF/IOA/meta_theory/Automata.thy	Wed May 21 11:27:32 1997 +0200
+++ b/src/HOLCF/IOA/meta_theory/Automata.thy	Wed May 21 15:08:52 1997 +0200
@@ -1,5 +1,5 @@
 (*  Title:      HOLCF/IOA/meta_theory/Automata.thy
-    ID:        
+    ID:         $Id$
     Author:     Olaf M"uller, Konrad Slind, Tobias Nipkow
     Copyright   1995, 1996  TU Muenchen
 
@@ -82,8 +82,8 @@
 
 state_trans_def
   "state_trans asig R == 
-    (!triple. triple:R --> fst(snd(triple)):actions(asig)) & 
-    (!a. (a:inputs(asig)) --> (!s1. ? s2. (s1,a,s2):R))"
+    (!triple. triple:R --> fst(snd(triple)):actions(asig))"
+(* & (!a. (a:inputs(asig)) --> (!s1. ? s2. (s1,a,s2):R))" *)
 
 
 asig_of_def   "asig_of == fst"