CookBook/Parsing.thy
changeset 114 13fd0a83d3c3
parent 108 8bea3f74889d
child 116 c9ff326e3ce5
equal deleted inserted replaced
113:9b6c9d172378 114:13fd0a83d3c3
   832   Below we change \isacommand{foobar} so that it takes a proposition as
   832   Below we change \isacommand{foobar} so that it takes a proposition as
   833   argument and then starts a proof in order to prove it. Therefore in Line 13, 
   833   argument and then starts a proof in order to prove it. Therefore in Line 13, 
   834   we set the kind indicator to @{ML thy_goal in OuterKeyword}.
   834   we set the kind indicator to @{ML thy_goal in OuterKeyword}.
   835 *}
   835 *}
   836 
   836 
   837 ML%linenumbers{*let
   837 ML%linenosgray{*let
   838   fun set_up_thm str ctxt =
   838   fun set_up_thm str ctxt =
   839     let
   839     let
   840       val prop = Syntax.read_prop ctxt str
   840       val prop = Syntax.read_prop ctxt str
   841     in
   841     in
   842       Proof.theorem_i NONE (K I) [[(prop,[])]] ctxt
   842       Proof.theorem_i NONE (K I) [[(prop,[])]] ctxt