ProgTutorial/FirstSteps.thy
changeset 378 8d160d79b48c
parent 377 272ba2cceeb2
child 385 78c91a629602
equal deleted inserted replaced
377:272ba2cceeb2 378:8d160d79b48c
   951 
   951 
   952   which shows the internal representation of the term @{text "Suc ?x"}. Similarly
   952   which shows the internal representation of the term @{text "Suc ?x"}. Similarly
   953   we can write an antiquotation for type patterns.
   953   we can write an antiquotation for type patterns.
   954 *}
   954 *}
   955 
   955 
   956 ML %linenosgray{*let
   956 ML{*let
   957   val parser = Args.context -- Scan.lift Args.name_source
   957   val parser = Args.context -- Scan.lift Args.name_source
   958 
   958 
   959   fun typ_pat (ctxt, str) =
   959   fun typ_pat (ctxt, str) =
   960      str |> Syntax.parse_typ ctxt
   960      str |> Syntax.parse_typ ctxt
   961          |> ML_Syntax.print_typ
   961          |> ML_Syntax.print_typ