src/Doc/Codegen/Further.thy
changeset 70022 49e178cbf923
parent 69697 4d95261fab5a
child 75074 78c2a92a8be4
equal deleted inserted replaced
70021:e6e634836556 70022:49e178cbf923
    46 code_reflect %quote Rat
    46 code_reflect %quote Rat
    47   datatypes rat
    47   datatypes rat
    48   functions Fract
    48   functions Fract
    49     "(plus :: rat \<Rightarrow> rat \<Rightarrow> rat)" "(minus :: rat \<Rightarrow> rat \<Rightarrow> rat)"
    49     "(plus :: rat \<Rightarrow> rat \<Rightarrow> rat)" "(minus :: rat \<Rightarrow> rat \<Rightarrow> rat)"
    50     "(times :: rat \<Rightarrow> rat \<Rightarrow> rat)" "(divide :: rat \<Rightarrow> rat \<Rightarrow> rat)"
    50     "(times :: rat \<Rightarrow> rat \<Rightarrow> rat)" "(divide :: rat \<Rightarrow> rat \<Rightarrow> rat)"
    51   file "$ISABELLE_TMP/rat.ML"
    51   file_prefix rat
    52 
    52 
    53 text \<open>
    53 text \<open>
    54   \noindent This merely generates the referenced code to the given
    54   \noindent This merely generates the referenced code to the given
    55   file which can be included into the system runtime later on.
    55   file which can be included into the system runtime later on.
    56 \<close>
    56 \<close>