src/Sequents/Sequents.thy
changeset 7121 0e3d09451b7a
parent 7098 86583034aacf
child 7166 a4a870ec2e67
equal deleted inserted replaced
7120:6d5923cecece 7121:0e3d09451b7a
    40  SeqContEmp     :: "seqcont"                            ("")
    40  SeqContEmp     :: "seqcont"                            ("")
    41  SeqContApp     :: "[seqobj,seqcont] => seqcont"        (",/ __")
    41  SeqContApp     :: "[seqobj,seqcont] => seqcont"        (",/ __")
    42   
    42   
    43  SeqO           :: "o => seqobj"                        ("_")
    43  SeqO           :: "o => seqobj"                        ("_")
    44  SeqId          :: "'a => seqobj"                       ("$_")
    44  SeqId          :: "'a => seqobj"                       ("$_")
    45  SeqVar         :: "var => seqobj"                      ("$_")
       
    46 
    45 
    47 types
    46 types
    48     
    47     
    49  single_seqe = "[seq,seqobj] => prop"
    48  single_seqe = "[seq,seqobj] => prop"
    50  single_seqi = "[seq'=>seq',seq'=>seq'] => prop"
    49  single_seqi = "[seq'=>seq',seq'=>seq'] => prop"