diff -r df053507edba -r 37285ec4387d Quot/Examples/LFex.thy --- a/Quot/Examples/LFex.thy Sun Dec 20 00:26:53 2009 +0100 +++ b/Quot/Examples/LFex.thy Sun Dec 20 00:53:35 2009 +0100 @@ -81,48 +81,48 @@ TRM = trm / atrm by (auto intro: alpha_equivps) -quotient_def +quotient_definition "TYP :: KIND" as "Type" -quotient_def +quotient_definition "KPI :: TY \ name \ KIND \ KIND" as "KPi" -quotient_def +quotient_definition "TCONST :: ident \ TY" as "TConst" -quotient_def +quotient_definition "TAPP :: TY \ TRM \ TY" as "TApp" -quotient_def +quotient_definition "TPI :: TY \ name \ TY \ TY" as "TPi" (* FIXME: does not work with CONST *) -quotient_def +quotient_definition "CONS :: ident \ TRM" as "Const" -quotient_def +quotient_definition "VAR :: name \ TRM" as "Var" -quotient_def +quotient_definition "APP :: TRM \ TRM \ TRM" as "App" -quotient_def +quotient_definition "LAM :: TY \ name \ TRM \ TRM" as "Lam" @@ -138,17 +138,17 @@ thm LAM_def (* FIXME: print out a warning if the type contains a liftet type, like kind \ name set *) -quotient_def +quotient_definition "FV_kind :: KIND \ name set" as "fv_kind" -quotient_def +quotient_definition "FV_ty :: TY \ name set" as "fv_ty" -quotient_def +quotient_definition "FV_trm :: TRM \ name set" as "fv_trm" @@ -164,17 +164,17 @@ perm_trm \ "perm :: 'x prm \ TRM \ TRM" (unchecked) begin -quotient_def +quotient_definition "perm_kind :: 'x prm \ KIND \ KIND" as "(perm::'x prm \ kind \ kind)" -quotient_def +quotient_definition "perm_ty :: 'x prm \ TY \ TY" as "(perm::'x prm \ ty \ ty)" -quotient_def +quotient_definition "perm_trm :: 'x prm \ TRM \ TRM" as "(perm::'x prm \ trm \ trm)"