doc-src/Codegen/Thy/Adaption.thy
changeset 30880 257cbe43faa8
parent 30836 1344132160bb
child 30882 d15725e84091
equal deleted inserted replaced
30879:efcba7788b2e 30880:257cbe43faa8
    53 *}
    53 *}
    54 
    54 
    55 subsection {* The adaption principle *}
    55 subsection {* The adaption principle *}
    56 
    56 
    57 text {*
    57 text {*
    58   The following figure illustrates what \qt{adaption} is conceptually
    58   Figure \ref{fig:adaption} illustrates what \qt{adaption} is conceptually
    59   supposed to be:
    59   supposed to be:
    60 
    60 
    61   \begin{figure}[here]
    61   \begin{figure}[here]
    62     \includegraphics{Thy/pictures/adaption}
    62     \includegraphics{Thy/pictures/adaption}
    63     \caption{The adaption principle}
    63     \caption{The adaption principle}
   285 
   285 
   286 definition %quote "eq_class.eq (x\<Colon>bar) y \<longleftrightarrow> x = y"
   286 definition %quote "eq_class.eq (x\<Colon>bar) y \<longleftrightarrow> x = y"
   287 
   287 
   288 instance %quote by default (simp add: eq_bar_def)
   288 instance %quote by default (simp add: eq_bar_def)
   289 
   289 
   290 end %quote
   290 end %quote (*<*)
   291 code_type %quotett bar
   291 
       
   292 (*>*) code_type %quotett bar
   292   (Haskell "Integer")
   293   (Haskell "Integer")
   293 
   294 
   294 text {*
   295 text {*
   295   \noindent The code generator would produce
   296   \noindent The code generator would produce
   296   an additional instance, which of course is rejected by the @{text Haskell}
   297   an additional instance, which of course is rejected by the @{text Haskell}