diff -r 75f7a77e53bb -r 9f906a2eb0e7 src/HOL/Quickcheck_Examples/Quickcheck_Nesting.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Quickcheck_Examples/Quickcheck_Nesting.thy Thu Sep 01 12:10:52 2016 +0200 @@ -0,0 +1,19 @@ +theory Quickcheck_Nesting +imports Main +begin + +ML \ +let + open BNF_FP_Def_Sugar + open BNF_LFP_Compat + + val compat_plugin = Plugin_Name.declare_setup @{binding compat}; + + fun compat fp_sugars = + perhaps (try (datatype_compat (map (fst o dest_Type o #T) fp_sugars))); +in + Theory.setup (fp_sugars_interpretation compat_plugin compat) +end +\ + +end