diff -r bfd9af005e23 -r 12ce01673188 Nominal/Test.thy --- a/Nominal/Test.thy Tue Mar 02 20:11:56 2010 +0100 +++ b/Nominal/Test.thy Tue Mar 02 20:14:21 2010 +0100 @@ -71,6 +71,8 @@ text {* example 1 *} +(* ML {* set show_hyps *} *) + nominal_datatype lam = VAR "name" | APP "lam" "lam" @@ -147,11 +149,13 @@ All xs::"name list" ty::"t_raw" bind xs in ty *) + +(* alpha_eqvt fails... nominal_datatype t = Var "name" | Fun "t" "t" and tyS = - All xs::"name set" ty::"t" bind xs in ty + All xs::"name set" ty::"t" bind xs in ty *) (* example 1 from Terms.thy *) @@ -205,6 +209,7 @@ (* example 4 from Terms.thy *) +(* fv_eqvt does not work, we need to repaire defined permute functions... nominal_datatype trm4 = Vr4 "name" | Ap4 "trm4" "trm4 list"