CookBook/Solutions.thy
changeset 156 e8f11280c762
parent 151 7e0bf13bf743
child 158 d7944bdf7b3f
equal deleted inserted replaced
155:b6fca043a796 156:e8f11280c762
     1 theory Solutions
     1 theory Solutions
     2 imports Base
     2 imports Base
     3 uses "infix_conv.ML"
     3 uses "infix_conv.ML"
     4 begin
     4 begin
     5 
     5 
     6 chapter {* Solutions to Most Exercises *}
     6 chapter {* Solutions to Most Exercises\label{ch:solutions} *}
     7 
     7 
     8 text {* \solution{fun:revsum} *}
     8 text {* \solution{fun:revsum} *}
     9 
     9 
    10 ML{*fun rev_sum t =
    10 ML{*fun rev_sum t =
    11 let
    11 let