src/HOL/IOA/ABP/Correctness.thy
changeset 1151 c820b3cc3df0
parent 1138 82fd99d5a6ff
child 1376 92f83b9d17e1
--- a/src/HOL/IOA/ABP/Correctness.thy	Wed Jun 21 15:14:58 1995 +0200
+++ b/src/HOL/IOA/ABP/Correctness.thy	Wed Jun 21 15:47:10 1995 +0200
@@ -19,12 +19,12 @@
 primrec
   reduce List.list  
   reduce_Nil  "reduce [] = []"
-  reduce_Cons "reduce(x#xs) =   \
-\	         (case xs of   \
-\	             [] => [x]   \
-\	       |   y#ys => (if (x=y)   \
-\	                      then reduce xs   \
-\	                      else (x#(reduce xs))))"
+  reduce_Cons "reduce(x#xs) =   
+	         (case xs of   
+	             [] => [x]   
+	       |   y#ys => (if (x=y)   
+	                      then reduce xs   
+	                      else (x#(reduce xs))))"
 
   
 defs
@@ -35,9 +35,9 @@
 system_fin_def
   "system_fin_ioa == (env_ioa || impl_fin_ioa)"
   
-abs_def "abs  ==   \
-\	(%p.(fst(p),(fst(snd(p)),(fst(snd(snd(p))),   \
-\	 (reduce(fst(snd(snd(snd(p))))),reduce(snd(snd(snd(snd(p))))))))))"
+abs_def "abs  ==   
+	(%p.(fst(p),(fst(snd(p)),(fst(snd(snd(p))),   
+	 (reduce(fst(snd(snd(snd(p))))),reduce(snd(snd(snd(snd(p))))))))))"
 
 rules
 
@@ -47,4 +47,3 @@
 end
 
 
-  
\ No newline at end of file