src/Sequents/LK0.thy
changeset 7166 a4a870ec2e67
parent 7118 ee384c7b7416
child 12116 4027b15377a5
equal deleted inserted replaced
7165:8c937127fd8c 7166:a4a870ec2e67
    21 
    21 
    22 consts
    22 consts
    23 
    23 
    24  Trueprop	:: "two_seqi"
    24  Trueprop	:: "two_seqi"
    25  "@Trueprop"	:: "two_seqe" ("((_)/ |- (_))" [6,6] 5)
    25  "@Trueprop"	:: "two_seqe" ("((_)/ |- (_))" [6,6] 5)
    26 
       
    27   (*Constant to allow definitions of SEQUENCES of formulas*)
       
    28   "@Side"        :: "seq=>(seq'=>seq')"     ("<<(_)>>")
       
    29 
    26 
    30   True,False   :: o
    27   True,False   :: o
    31   "="          :: ['a,'a] => o       (infixl 50)
    28   "="          :: ['a,'a] => o       (infixl 50)
    32   Not          :: o => o             ("~ _" [40] 40)
    29   Not          :: o => o             ("~ _" [40] 40)
    33   "&"          :: [o,o] => o         (infixr 35)
    30   "&"          :: [o,o] => o         (infixr 35)
   136 
   133 
   137 end
   134 end
   138 
   135 
   139 ML
   136 ML
   140 
   137 
   141 fun side_tr [s1] = Sequents.seq_tr s1;
       
   142 
   138 
   143 val parse_translation = [("@Trueprop",Sequents.two_seq_tr "Trueprop"),
   139 val parse_translation = [("@Trueprop",Sequents.two_seq_tr "Trueprop")];
   144 			 ("@Side", side_tr)];
       
   145 val print_translation = [("Trueprop",Sequents.two_seq_tr' "@Trueprop")];
   140 val print_translation = [("Trueprop",Sequents.two_seq_tr' "@Trueprop")];
   146 
   141