CookBook/Recipes/StoringData.thy
changeset 119 4536782969fa
parent 72 7b8c4fe235aa
equal deleted inserted replaced
118:5f003fdf2653 119:4536782969fa
     1 theory StoringData
     1 theory StoringData
     2 imports "../Base"
     2 imports "../Base"
     3 begin
     3 begin
     4 
     4 
     5 section {* Storing Data\label{recipe:storingdata} *} 
     5 section {* Storing Data\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