IOA/meta_theory/Asig.thy
changeset 249 492493334e0f
parent 168 44ff2275d44f
--- a/IOA/meta_theory/Asig.thy	Fri Apr 14 11:23:33 1995 +0200
+++ b/IOA/meta_theory/Asig.thy	Wed Jun 21 15:12:40 1995 +0200
@@ -32,10 +32,10 @@
    "externals(asig) == (inputs(asig) Un outputs(asig))"
 
 is_asig_def
-  "is_asig(triple) ==            \
-   \  ((inputs(triple) Int outputs(triple) = {})    & \
-   \   (outputs(triple) Int internals(triple) = {}) & \
-   \   (inputs(triple) Int internals(triple) = {}))"
+  "is_asig(triple) ==            
+      ((inputs(triple) Int outputs(triple) = {})    & 
+       (outputs(triple) Int internals(triple) = {}) & 
+       (inputs(triple) Int internals(triple) = {}))"
 
 
 mk_ext_asig_def