src/Doc/Codegen/Introduction.thy
changeset 59378 065f349852e6
parent 59377 056945909f60
child 61076 bdc1e2f0a86a
equal deleted inserted replaced
59377:056945909f60 59378:065f349852e6
     1 theory Introduction
     1 theory Introduction
     2 imports Setup
     2 imports Setup
     3 begin
     3 begin (*<*)
       
     4 
       
     5 ML \<open>
       
     6   Isabelle_System.mkdirs (File.tmp_path (Path.basic "examples"))
       
     7 \<close> (*>*)
     4 
     8 
     5 section \<open>Introduction\<close>
     9 section \<open>Introduction\<close>
     6 
    10 
     7 text \<open>
    11 text \<open>
     8   This tutorial introduces the code generator facilities of @{text
    12   This tutorial introduces the code generator facilities of @{text