doc-src/Codegen/Thy/Adaptation.thy
changeset 38506 03d767575713
parent 38505 2f8699695cf6
child 39063 5f9692dd621f
equal deleted inserted replaced
38505:2f8699695cf6 38506:03d767575713
   305   (Haskell "Integer")
   305   (Haskell "Integer")
   306 
   306 
   307 text {*
   307 text {*
   308   \noindent The code generator would produce an additional instance,
   308   \noindent The code generator would produce an additional instance,
   309   which of course is rejected by the @{text Haskell} compiler.  To
   309   which of course is rejected by the @{text Haskell} compiler.  To
   310   suppress this additional instance, use @{text "code_instance"}:
   310   suppress this additional instance, use @{command_def "code_instance"}:
   311 *}
   311 *}
   312 
   312 
   313 code_instance %quotett bar :: eq
   313 code_instance %quotett bar :: eq
   314   (Haskell -)
   314   (Haskell -)
   315 
   315