ProgTutorial/Base.thy
changeset 255 ef1da1abee46
parent 239 b63c72776f03
child 256 1fb8d62c88a0
equal deleted inserted replaced
254:cb86bf5658e4 255:ef1da1abee46
     1 theory Base
     1 theory Base
     2 imports Main
     2 imports Main
     3 uses
     3 uses
       
     4   "outputfn.ML"
     4   "chunks.ML"
     5   "chunks.ML"
     5   "antiquote_setup.ML"
     6   "antiquote_setup.ML"
     6 begin
     7 begin
     7 
     8 
     8 (* to have a special tag for text enclosed in ML *)
     9 (* to have a special tag for text enclosed in ML *)
    35   (OuterKeyword.tag "TutorialML" OuterKeyword.diag)
    36   (OuterKeyword.tag "TutorialML" OuterKeyword.diag)
    36     (OuterParse.ML_source >> IsarCmd.ml_diag true);
    37     (OuterParse.ML_source >> IsarCmd.ml_diag true);
    37 
    38 
    38 *}
    39 *}
    39 
    40 
       
    41 
    40 end
    42 end