ProgTutorial/Base.thy
changeset 419 2e199c5faf76
parent 396 a2e49e0771b3
child 423 0a25b35178c3
equal deleted inserted replaced
418:1d1e4cda8c54 419:2e199c5faf76
    18 (* re-definition of various ML antiquotations     *)
    18 (* re-definition of various ML antiquotations     *)
    19 (* to have a special tag for text enclosed in ML; *)
    19 (* to have a special tag for text enclosed in ML; *)
    20 (* they also write the code into a separate file  *)
    20 (* they also write the code into a separate file  *)
    21 
    21 
    22 ML {*
    22 ML {*
    23 val (filename, setup_filename) = Attrib.config_string "filename" "File_Code.ML"
    23 val (filename, setup_filename) = Attrib.config_string "filename" (K "File_Code.ML")
    24 *}
    24 *}
    25 
    25 
    26 setup {* setup_filename *}
    26 setup {* setup_filename *}
    27 
    27 
    28 ML {*
    28 ML {*