diff -r fdbea66eae4b -r 17e29ddd538e src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy --- a/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Thu Sep 30 10:48:12 2010 +0200 +++ b/src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy Thu Sep 30 10:48:12 2010 +0200 @@ -100,6 +100,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_predicates = [(["repIntPa"], 2), (["repP"], 2), (["subP"], 0), (["accepts", "acceptsaux", "seqSplit", "seqSplita", "seqSplitaux", "seqSplitb"], 25)],