src/Doc/Codegen/Introduction.thy
changeset 65981 e2c25346b156
parent 61076 bdc1e2f0a86a
child 66453 cc19f7ca2ed6
equal deleted inserted replaced
65980:3bec939bd808 65981:e2c25346b156
    68   by (cases xs) (simp_all split: list.splits) (*>*)
    68   by (cases xs) (simp_all split: list.splits) (*>*)
    69 
    69 
    70 text \<open>\noindent Then we can generate code e.g.~for @{text SML} as follows:\<close>
    70 text \<open>\noindent Then we can generate code e.g.~for @{text SML} as follows:\<close>
    71 
    71 
    72 export_code %quote empty dequeue enqueue in SML
    72 export_code %quote empty dequeue enqueue in SML
    73   module_name Example file "$ISABELLE_TMP/examples/example.ML"
    73   module_name Example file "$ISABELLE_TMP/example.ML"
    74 
    74 
    75 text \<open>\noindent resulting in the following code:\<close>
    75 text \<open>\noindent resulting in the following code:\<close>
    76 
    76 
    77 text %quotetypewriter \<open>
    77 text %quotetypewriter \<open>
    78   @{code_stmts empty enqueue dequeue (SML)}
    78   @{code_stmts empty enqueue dequeue (SML)}