src/HOL/IOA/meta_theory/IOA.thy
changeset 1476 608483c2122a
parent 1151 c820b3cc3df0
child 2018 bcd69cc47cf0
--- a/src/HOL/IOA/meta_theory/IOA.thy	Mon Feb 05 21:27:16 1996 +0100
+++ b/src/HOL/IOA/meta_theory/IOA.thy	Mon Feb 05 21:29:06 1996 +0100
@@ -22,7 +22,7 @@
   asig_of    ::"('action,'state)ioa => 'action signature"
   starts_of  ::"('action,'state)ioa => 'state set"
   trans_of   ::"('action,'state)ioa => ('action,'state)transition set"
-  IOA	     ::"('action,'state)ioa => bool"
+  IOA        ::"('action,'state)ioa => bool"
 
   (* Executions, schedules, and traces *)