diff -r 4e586b734fac -r 3aa2bc9c5478 doc-src/Codegen/Thy/Adaptation.thy --- a/doc-src/Codegen/Thy/Adaptation.thy Mon Sep 27 16:19:37 2010 +0200 +++ b/doc-src/Codegen/Thy/Adaptation.thy Mon Sep 27 16:27:31 2010 +0200 @@ -175,7 +175,7 @@ code_const %invisible True and False and "op \" and Not (SML and and and) (*>*) -text %quote %typewriter {* +text %quotetypewriter {* @{code_stmts in_interval (SML)} *} @@ -190,9 +190,9 @@ "bool"}, we may use \qn{custom serialisations}: *} -code_type %quote %tt bool +code_type %quotett bool (SML "bool") -code_const %quote %tt True and False and "op \" +code_const %quotett True and False and "op \" (SML "true" and "false" and "_ andalso _") text {* @@ -206,7 +206,7 @@ placeholder for the type constructor's (the constant's) arguments. *} -text %quote %typewriter {* +text %quotetypewriter {* @{code_stmts in_interval (SML)} *} @@ -218,10 +218,10 @@ precedences which may be used here: *} -code_const %quote %tt "op \" +code_const %quotett "op \" (SML infixl 1 "andalso") -text %quote %typewriter {* +text %quotetypewriter {* @{code_stmts in_interval (SML)} *} @@ -247,9 +247,9 @@ code_const %invisible Pair (SML) (*>*) -code_type %quote %tt prod +code_type %quotett prod (SML infix 2 "*") -code_const %quote %tt Pair +code_const %quotett Pair (SML "!((_),/ (_))") text {* @@ -283,10 +283,10 @@ @{command_def code_class}) and its operation @{const [source] HOL.equal} *} -code_class %quote %tt equal +code_class %quotett equal (Haskell "Eq") -code_const %quote %tt "HOL.equal" +code_const %quotett "HOL.equal" (Haskell infixl 4 "==") text {* @@ -307,7 +307,7 @@ end %quote (*<*) -(*>*) code_type %quote %tt bar +(*>*) code_type %quotett bar (Haskell "Integer") text {* @@ -316,7 +316,7 @@ suppress this additional instance, use @{command_def "code_instance"}: *} -code_instance %quote %tt bar :: equal +code_instance %quotett bar :: equal (Haskell -) @@ -328,10 +328,10 @@ "code_include"} command: *} -code_include %quote %tt Haskell "Errno" +code_include %quotett Haskell "Errno" {*errno i = error ("Error number: " ++ show i)*} -code_reserved %quote %tt Haskell Errno +code_reserved %quotett Haskell Errno text {* \noindent Such named @{text include}s are then prepended to every