diff -r e3bbc2c4c581 -r 20d01210b9b1 src/HOL/Predicate.thy --- a/src/HOL/Predicate.thy Mon Apr 20 12:27:23 2009 +0200 +++ b/src/HOL/Predicate.thy Mon Apr 20 16:28:13 2009 +0200 @@ -622,6 +622,31 @@ "pred_rec f P = f (eval P)" by (cases P) simp +export_code Seq in Eval module_name Predicate + +ML {* +signature PREDICATE = +sig + datatype 'a pred = Seq of (unit -> 'a seq) + and 'a seq = Empty | Insert of 'a * 'a pred | Join of 'a pred * 'a seq +end; + +structure Predicate : PREDICATE = +struct + +open Predicate; + +end; +*} + +code_reserved Eval Predicate + +code_type pred and seq + (Eval "_/ Predicate.pred" and "_/ Predicate.seq") + +code_const Seq and Empty and Insert and Join + (Eval "Predicate.Seq" and "Predicate.Empty" and "Predicate.Insert/ (_,/ _)" and "Predicate.Join/ (_,/ _)") + no_notation inf (infixl "\" 70) and sup (infixl "\" 65) and