ProgTutorial/FirstSteps.thy
changeset 326 f76135c6c527
parent 325 352e31d9dacc
child 327 ce754ad78bc9
equal deleted inserted replaced
325:352e31d9dacc 326:f76135c6c527
   883 
   883 
   884 ML {*
   884 ML {*
   885  project_bool (nth list 1)
   885  project_bool (nth list 1)
   886 *}
   886 *}
   887 
   887 
       
   888 ML {* 
       
   889   Context.the_thread_data ();
       
   890   Context.display_names @{theory};
       
   891   Context.pretty_thy @{theory}
       
   892     |> Pretty.string_of
       
   893     |> tracing
       
   894 *}
       
   895 
       
   896 text {*
       
   897   \begin{readmore}
       
   898   @{ML_file "Pure/ML-Systems/universal.ML"}
       
   899   \end{readmore}
       
   900 *}
       
   901 
   888 (**************************************************)
   902 (**************************************************)
   889 (* bak                                            *)
   903 (* bak                                            *)
   890 (**************************************************)
   904 (**************************************************)
   891 
   905 
   892 (*
   906 (*