src/HOL/ex/Simult.thy
changeset 1381 57777949b2f8
parent 1376 92f83b9d17e1
child 1476 608483c2122a
equal deleted inserted replaced
1380:2f8055af9c04 1381:57777949b2f8
    29   Rep_Forest  :: 'a forest => 'a item
    29   Rep_Forest  :: 'a forest => 'a item
    30   Abs_Forest  :: 'a item => 'a forest
    30   Abs_Forest  :: 'a item => 'a forest
    31   Tcons       :: ['a, 'a forest] => 'a tree
    31   Tcons       :: ['a, 'a forest] => 'a tree
    32   Fcons       :: ['a tree, 'a forest] => 'a forest
    32   Fcons       :: ['a tree, 'a forest] => 'a forest
    33   Fnil        :: 'a forest
    33   Fnil        :: 'a forest
    34   TF_rec      :: "['a item, ['a item , 'a item, 'b]=>'b,     
    34   TF_rec      :: ['a item, ['a item , 'a item, 'b]=>'b,     
    35                  'b, ['a item , 'a item, 'b, 'b]=>'b] => 'b"
    35                  'b, ['a item , 'a item, 'b, 'b]=>'b] => 'b
    36   tree_rec    :: "['a tree, ['a, 'a forest, 'b]=>'b,          
    36   tree_rec    :: ['a tree, ['a, 'a forest, 'b]=>'b,          
    37                  'b, ['a tree, 'a forest, 'b, 'b]=>'b] => 'b"
    37                  'b, ['a tree, 'a forest, 'b, 'b]=>'b] => 'b
    38   forest_rec  :: "['a forest, ['a, 'a forest, 'b]=>'b,        
    38   forest_rec  :: ['a forest, ['a, 'a forest, 'b]=>'b,        
    39                   'b, ['a tree, 'a forest, 'b, 'b]=>'b] => 'b"
    39                   'b, ['a tree, 'a forest, 'b, 'b]=>'b] => 'b
    40 
    40 
    41 defs
    41 defs
    42      (*the concrete constants*)
    42      (*the concrete constants*)
    43   TCONS_def 	"TCONS M N == In0(M $ N)"
    43   TCONS_def 	"TCONS M N == In0(M $ N)"
    44   FNIL_def	"FNIL      == In1(NIL)"
    44   FNIL_def	"FNIL      == In1(NIL)"