diff -r c8a2755bf220 -r ff784d5a5bfb src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy --- a/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Sat Jan 05 17:24:33 2019 +0100 @@ -106,7 +106,7 @@ setup \Code_Prolog.map_code_options (K {ensure_groundness = true, limit_globally = NONE, - limited_types = [(@{typ Sym}, 0), (@{typ "Sym list"}, 2), (@{typ RE}, 6)], + limited_types = [(\<^typ>\Sym\, 0), (\<^typ>\Sym list\, 2), (\<^typ>\RE\, 6)], limited_predicates = [(["repIntPa"], 2), (["repP"], 2), (["subP"], 0), (["accepts", "acceptsaux", "seqSplit", "seqSplita", "seqSplitaux", "seqSplitb"], 25)], replacing =