ProgTutorial/Recipes/StoringData.thy
changeset 211 d5accbc67e1b
parent 189 069d525f8f1d
equal deleted inserted replaced
210:db8e302f44c8 211:d5accbc67e1b
     1 theory StoringData
     1 theory StoringData
     2 imports "../Base"
     2 imports "../Base"
     3 begin
     3 begin
     4 
     4 
     5 section {* Storing Data\label{rec:storingdata} *} 
     5 section {* Storing Data (TBD)\label{rec:storingdata} *} 
     6 
     6 
     7 
     7 
     8 text {*
     8 text {*
     9   {\bf Problem:} 
     9   {\bf Problem:} 
    10   Your tool needs to manage data.\smallskip
    10   Your tool needs to manage data.\smallskip