src/Pure/Isar/isar_syn.ML
changeset 37198 3af985b10550
parent 36953 2af1ad9aa1a3
child 37216 3165bc303f66
equal deleted inserted replaced
37197:953fc4983439 37198:3af985b10550
   319 val _ =
   319 val _ =
   320   Outer_Syntax.command "ML" "ML text within theory or local theory"
   320   Outer_Syntax.command "ML" "ML text within theory or local theory"
   321     (Keyword.tag_ml Keyword.thy_decl)
   321     (Keyword.tag_ml Keyword.thy_decl)
   322     (Parse.ML_source >> (fn (txt, pos) =>
   322     (Parse.ML_source >> (fn (txt, pos) =>
   323       Toplevel.generic_theory
   323       Toplevel.generic_theory
   324         (ML_Context.exec (fn () => ML_Context.eval true pos txt) #> propagate_env)));
   324         (ML_Context.exec (fn () => ML_Context.eval_text true pos txt) #> propagate_env)));
   325 
   325 
   326 val _ =
   326 val _ =
   327   Outer_Syntax.command "ML_prf" "ML text within proof" (Keyword.tag_proof Keyword.prf_decl)
   327   Outer_Syntax.command "ML_prf" "ML text within proof" (Keyword.tag_proof Keyword.prf_decl)
   328     (Parse.ML_source >> (fn (txt, pos) =>
   328     (Parse.ML_source >> (fn (txt, pos) =>
   329       Toplevel.proof (Proof.map_context (Context.proof_map
   329       Toplevel.proof (Proof.map_context (Context.proof_map
   330         (ML_Context.exec (fn () => ML_Context.eval true pos txt))) #> propagate_env_prf)));
   330         (ML_Context.exec (fn () => ML_Context.eval_text true pos txt))) #> propagate_env_prf)));
   331 
   331 
   332 val _ =
   332 val _ =
   333   Outer_Syntax.command "ML_val" "diagnostic ML text" (Keyword.tag_ml Keyword.diag)
   333   Outer_Syntax.command "ML_val" "diagnostic ML text" (Keyword.tag_ml Keyword.diag)
   334     (Parse.ML_source >> IsarCmd.ml_diag true);
   334     (Parse.ML_source >> IsarCmd.ml_diag true);
   335 
   335