fixed title line; added spacing
authorpaulson
Fri, 11 Jun 1999 10:35:55 +0200
changeset 6819 433a980103b4
parent 6818 852f9ed01a53
child 6820 41d9b7bbf968
fixed title line; added spacing
src/Sequents/Sequents.thy
--- a/src/Sequents/Sequents.thy	Fri Jun 11 10:34:20 1999 +0200
+++ b/src/Sequents/Sequents.thy	Fri Jun 11 10:35:55 1999 +0200
@@ -1,4 +1,4 @@
-(*  Title: 	LK/lk.thy
+(*  Title: 	Sequents/Sequents.thy
     ID:         $Id$
     Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1993  University of Cambridge
@@ -61,20 +61,20 @@
 
 fun abs_seq' t = Abs("s", Type("seq'",[]), t);
 
-fun seqobj_tr(Const("SeqO",_)$f) = Const("SeqO'",dummyT)$f |
-    seqobj_tr(_$i) = i;
+fun seqobj_tr(Const("SeqO",_) $ f) = Const("SeqO'",dummyT) $ f |
+    seqobj_tr(_ $ i) = i;
     
 fun seqcont_tr(Const("SeqContEmp",_)) = Bound 0 |
-    seqcont_tr(Const("SeqContApp",_)$so$sc) = 
-      (seqobj_tr so)$(seqcont_tr sc);
+    seqcont_tr(Const("SeqContApp",_) $ so $ sc) = 
+      (seqobj_tr so) $ (seqcont_tr sc);
 
 fun seq_tr(Const("SeqEmp",_)) = abs_seq'(Bound 0) |
-    seq_tr(Const("SeqApp",_)$so$sc) = 
-      abs_seq'(seqobj_tr(so)$seqcont_tr(sc));
+    seq_tr(Const("SeqApp",_) $ so $ sc) = 
+      abs_seq'(seqobj_tr(so) $ seqcont_tr(sc));
 
 
-fun singlobj_tr(Const("SeqO",_)$f) =
-    abs_seq' ((Const("SeqO'",dummyT)$f)$Bound 0);
+fun singlobj_tr(Const("SeqO",_) $ f) =
+    abs_seq' ((Const("SeqO'",dummyT) $ f) $ Bound 0);
     
 
     
@@ -82,66 +82,66 @@
 
 fun seqcont_tr' (Bound 0) = 
       Const("SeqContEmp",dummyT) |
-    seqcont_tr' (Const("SeqO'",_)$f$s) =
-      Const("SeqContApp",dummyT)$
-      (Const("SeqO",dummyT)$f)$
+    seqcont_tr' (Const("SeqO'",_) $ f $ s) =
+      Const("SeqContApp",dummyT) $ 
+      (Const("SeqO",dummyT) $ f) $ 
       (seqcont_tr' s) |
-(*    seqcont_tr' ((a as Abs(_,_,_))$s)= 
+(*    seqcont_tr' ((a as Abs(_,_,_)) $ s)= 
       seqcont_tr'(betapply(a,s)) | *)
-    seqcont_tr' (i$s) = 
-      Const("SeqContApp",dummyT)$
-      (Const("SeqId",dummyT)$i)$
+    seqcont_tr' (i $ s) = 
+      Const("SeqContApp",dummyT) $ 
+      (Const("SeqId",dummyT) $ i) $ 
       (seqcont_tr' s);
 
 fun seq_tr' s =
     let fun seq_itr' (Bound 0) = 
               Const("SeqEmp",dummyT) |
-            seq_itr' (Const("SeqO'",_)$f$s) =
-              Const("SeqApp",dummyT)$
-              (Const("SeqO",dummyT)$f)$(seqcont_tr' s) |
-(*            seq_itr' ((a as Abs(_,_,_))$s) =
+            seq_itr' (Const("SeqO'",_) $ f $ s) =
+              Const("SeqApp",dummyT) $ 
+              (Const("SeqO",dummyT) $ f) $ (seqcont_tr' s) |
+(*            seq_itr' ((a as Abs(_,_,_)) $ s) =
               seq_itr'(betapply(a,s)) |    *)
-            seq_itr' (i$s) =
-              Const("SeqApp",dummyT)$
-              (Const("SeqId",dummyT)$i)$
+            seq_itr' (i $ s) =
+              Const("SeqApp",dummyT) $ 
+              (Const("SeqId",dummyT) $ i) $ 
               (seqcont_tr' s)
     in case s of 
          Abs(_,_,t) => seq_itr' t |
-         _ => s$(Bound 0)
+         _ => s $ (Bound 0)
     end;
 
 
 
 
 fun single_tr c [s1,s2] =
-    Const(c,dummyT)$seq_tr s1$singlobj_tr s2;
+    Const(c,dummyT) $ seq_tr s1 $ singlobj_tr s2;
 
 fun two_seq_tr c [s1,s2] =
-    Const(c,dummyT)$seq_tr s1$seq_tr s2;
+    Const(c,dummyT) $ seq_tr s1 $ seq_tr s2;
 
 fun three_seq_tr c [s1,s2,s3] =
-    Const(c,dummyT)$seq_tr s1$seq_tr s2$seq_tr s3;
+    Const(c,dummyT) $ seq_tr s1 $ seq_tr s2 $ seq_tr s3;
 
 fun four_seq_tr c [s1,s2,s3,s4] =
-    Const(c,dummyT)$seq_tr s1$seq_tr s2$seq_tr s3$seq_tr s4;
+    Const(c,dummyT) $ seq_tr s1 $ seq_tr s2 $ seq_tr s3 $ seq_tr s4;
 
 
-fun singlobj_tr'(Const("SeqO'",_)$fm) = fm |
-    singlobj_tr'(id) = Const("@SeqId",dummyT)$id;
+fun singlobj_tr'(Const("SeqO'",_) $ fm) = fm |
+    singlobj_tr'(id) = Const("@SeqId",dummyT) $ id;
 
 
 fun single_tr' c [s1, s2] =
-(Const (c, dummyT)$seq_tr' s1$seq_tr' s2 ); 
+(Const (c, dummyT) $ seq_tr' s1 $ seq_tr' s2 ); 
 
 
 fun two_seq_tr' c [s1, s2] =
-  Const (c, dummyT)$seq_tr' s1$seq_tr' s2; 
+  Const (c, dummyT) $ seq_tr' s1 $ seq_tr' s2; 
 
 fun three_seq_tr' c [s1, s2, s3] =
-  Const (c, dummyT)$seq_tr' s1$seq_tr' s2$seq_tr' s3; 
+  Const (c, dummyT) $ seq_tr' s1 $ seq_tr' s2 $ seq_tr' s3; 
 
 fun four_seq_tr' c [s1, s2, s3, s4] =
-  Const (c, dummyT)$seq_tr' s1$seq_tr' s2$seq_tr' s3$seq_tr' s4; 
+  Const (c, dummyT) $ seq_tr' s1 $ seq_tr' s2 $ seq_tr' s3 $ seq_tr' s4;