QuotMain.thy
changeset 205 2a803a1556d5
parent 203 7384115df9fd
child 207 18d7d9dc75cb
child 212 ca9eae5bd871
equal deleted inserted replaced
204:524e0e9cf6b6 205:2a803a1556d5
   150 ML {* maps_lookup @{theory} "fun" *}
   150 ML {* maps_lookup @{theory} "fun" *}
   151 
   151 
   152 ML {*
   152 ML {*
   153 val quot_def_parser = 
   153 val quot_def_parser = 
   154   (OuterParse.$$$ "(" |-- OuterParse.$$$ "with" |-- 
   154   (OuterParse.$$$ "(" |-- OuterParse.$$$ "with" |-- 
   155     ((OuterParse.list1 OuterParse.binding) --| OuterParse.$$$ ")")) --
   155     ((OuterParse.list1 OuterParse.typ) --| OuterParse.$$$ ")")) --
   156       (OuterParse.binding -- 
   156       (OuterParse.binding -- 
   157         Scan.option (OuterParse.$$$ "::" |-- OuterParse.typ) -- 
   157         Scan.option (OuterParse.$$$ "::" |-- OuterParse.typ) -- 
   158          OuterParse.mixfix --| OuterParse.where_ -- SpecParse.spec)
   158          OuterParse.mixfix --| OuterParse.where_ -- SpecParse.spec)
   159 *}
   159 *}
   160 
   160