diff -r 0fd4abb5fade -r f51c6069cd17 Quot/Examples/LFex.thy --- a/Quot/Examples/LFex.thy Fri Dec 11 08:28:41 2009 +0100 +++ b/Quot/Examples/LFex.thy Fri Dec 11 11:08:58 2009 +0100 @@ -81,49 +81,49 @@ by (auto intro: alpha_equivps) quotient_def - TYP :: "TYP :: KIND" -where + "TYP :: KIND" +as "Type" quotient_def - KPI :: "KPI :: TY \ name \ KIND \ KIND" -where + "KPI :: TY \ name \ KIND \ KIND" +as "KPi" quotient_def - TCONST :: "TCONST :: ident \ TY" -where + "TCONST :: ident \ TY" +as "TConst" quotient_def - TAPP :: "TAPP :: TY \ TRM \ TY" -where + "TAPP :: TY \ TRM \ TY" +as "TApp" quotient_def - TPI :: "TPI :: TY \ name \ TY \ TY" -where + "TPI :: TY \ name \ TY \ TY" +as "TPi" (* FIXME: does not work with CONST *) quotient_def - CONS :: "CONS :: ident \ TRM" -where + "CONS :: ident \ TRM" +as "Const" quotient_def - VAR :: "VAR :: name \ TRM" -where + "VAR :: name \ TRM" +as "Var" quotient_def - APP :: "APP :: TRM \ TRM \ TRM" -where + "APP :: TRM \ TRM \ TRM" +as "App" quotient_def - LAM :: "LAM :: TY \ name \ TRM \ TRM" -where + "LAM :: TY \ name \ TRM \ TRM" +as "Lam" thm TYP_def @@ -138,18 +138,18 @@ (* FIXME: print out a warning if the type contains a liftet type, like kind \ name set *) quotient_def - FV_kind :: "FV_kind :: KIND \ name set" -where + "FV_kind :: KIND \ name set" +as "fv_kind" quotient_def - FV_ty :: "FV_ty :: TY \ name set" -where + "FV_ty :: TY \ name set" +as "fv_ty" quotient_def - FV_trm :: "FV_trm :: TRM \ name set" -where + "FV_trm :: TRM \ name set" +as "fv_trm" thm FV_kind_def @@ -164,18 +164,18 @@ begin quotient_def - perm_kind :: "perm_kind :: 'x prm \ KIND \ KIND" -where + "perm_kind :: 'x prm \ KIND \ KIND" +as "(perm::'x prm \ kind \ kind)" quotient_def - perm_ty :: "perm_ty :: 'x prm \ TY \ TY" -where + "perm_ty :: 'x prm \ TY \ TY" +as "(perm::'x prm \ ty \ ty)" quotient_def - perm_trm :: "perm_trm :: 'x prm \ TRM \ TRM" -where + "perm_trm :: 'x prm \ TRM \ TRM" +as "(perm::'x prm \ trm \ trm)" end