ProgTutorial/Solutions.thy
changeset 441 520127b708e6
parent 440 a0b280dd4bc7
child 446 4c32349b9875
equal deleted inserted replaced
440:a0b280dd4bc7 441:520127b708e6
     1 theory Solutions
     1 theory Solutions
     2 imports FirstSteps "Recipes/Timing"
     2 imports First_Steps "Recipes/Timing"
     3 begin
     3 begin
     4 
     4 
     5 (*<*)
     5 (*<*)
     6 setup{*
     6 setup{*
     7 open_file_with_prelude 
     7 open_file_with_prelude 
     8   "Solutions_Code.thy"
     8   "Solutions_Code.thy"
     9   ["theory Solutions", "imports FirstSteps", "begin"]
     9   ["theory Solutions", "imports First_Steps", "begin"]
    10 *}
    10 *}
    11 (*>*)
    11 (*>*)
    12 
    12 
    13 chapter {* Solutions to Most Exercises\label{ch:solutions} *}
    13 chapter {* Solutions to Most Exercises\label{ch:solutions} *}
    14 
    14