src/HOL/ex/Simult.thy
changeset 2911 8a680e310f04
parent 1476 608483c2122a
equal deleted inserted replaced
2910:905aa895136c 2911:8a680e310f04
    70                (%g. Case (Split(%x y. b x y (g y))) 
    70                (%g. Case (Split(%x y. b x y (g y))) 
    71                       (List_case c (%x y. d x y (g x) (g y)))) M"
    71                       (List_case c (%x y. d x y (g x) (g y)))) M"
    72 
    72 
    73   tree_rec_def
    73   tree_rec_def
    74    "tree_rec t b c d == 
    74    "tree_rec t b c d == 
    75    TF_rec (Rep_Tree t) (%x y r. b (Inv Leaf x) (Abs_Forest y) r) 
    75    TF_rec (Rep_Tree t) (%x y r. b (inv Leaf x) (Abs_Forest y) r) 
    76           c (%x y rt rf. d (Abs_Tree x) (Abs_Forest y) rt rf)"
    76           c (%x y rt rf. d (Abs_Tree x) (Abs_Forest y) rt rf)"
    77 
    77 
    78   forest_rec_def
    78   forest_rec_def
    79    "forest_rec tf b c d == 
    79    "forest_rec tf b c d == 
    80    TF_rec (Rep_Forest tf) (%x y r. b (Inv Leaf x) (Abs_Forest y) r) 
    80    TF_rec (Rep_Forest tf) (%x y r. b (inv Leaf x) (Abs_Forest y) r) 
    81           c (%x y rt rf. d (Abs_Tree x) (Abs_Forest y) rt rf)"
    81           c (%x y rt rf. d (Abs_Tree x) (Abs_Forest y) rt rf)"
    82 end
    82 end