ProgTutorial/Solutions.thy
changeset 346 0fea8b7a14a1
parent 329 5dffcab68680
child 351 f118240ab44a
equal deleted inserted replaced
345:4c54ef4dc84d 346:0fea8b7a14a1
     1 theory Solutions
     1 theory Solutions
     2 imports FirstSteps "Recipes/Timing"
     2 imports FirstSteps "Recipes/Timing"
     3 begin
     3 begin
       
     4 
       
     5 (*<*)
       
     6 setup{*
       
     7 open_file_with_prelude 
       
     8   "Solutions_Code.thy"
       
     9   ["theory Solutions", "imports FirstSteps", "begin"]
       
    10 *}
       
    11 (*>*)
     4 
    12 
     5 chapter {* Solutions to Most Exercises\label{ch:solutions} *}
    13 chapter {* Solutions to Most Exercises\label{ch:solutions} *}
     6 
    14 
     7 text {* \solution{fun:revsum} *}
    15 text {* \solution{fun:revsum} *}
     8 
    16