diff -r 112eefe85ff0 -r 532ad8de5d61 src/Doc/Datatypes/Datatypes.thy --- a/src/Doc/Datatypes/Datatypes.thy Wed Feb 17 12:07:49 2016 +0100 +++ b/src/Doc/Datatypes/Datatypes.thy Wed Feb 17 11:39:26 2016 +0100 @@ -359,7 +359,7 @@ Cons (infixr "#" 65) hide_type list - hide_const Nil Cons case_list hd tl set map list_all2 rec_list size_list pred_list + hide_const Nil Cons case_list hd tl set map list_all2 rec_list size_list list_all context early begin @@ -370,6 +370,7 @@ for map: map rel: list_all2 + pred: list_all where "tl Nil = Nil" @@ -439,6 +440,7 @@ for map: map rel: list_all2 + pred: list_all text \ \noindent @@ -2889,7 +2891,7 @@ lift_bnf (*<*)(no_warn_wits) (*>*)'a nonempty_list proof - - fix f and xs :: "'a list" + fix f(*<*):: "'a \ 'c"(*>*) and xs :: "'a list" assume "xs \ {xs. xs \ []}" then show "map f xs \ {xs. xs \ []}" by (cases xs(*<*) rule: list.exhaust(*>*)) auto