equal
  deleted
  inserted
  replaced
  
    
    
|      6  |      6  | 
|      7 atom_decl var |      7 atom_decl var | 
|      8 atom_decl cvar |      8 atom_decl cvar | 
|      9 atom_decl tvar |      9 atom_decl tvar | 
|     10  |     10  | 
|     11 declare [[STEPS = 4]] |     11 declare [[STEPS = 9]] | 
|     12  |     12  | 
|     13 nominal_datatype tkind = |     13 nominal_datatype tkind = | 
|     14   KStar |     14   KStar | 
|     15 | KFun "tkind" "tkind" |     15 | KFun "tkind" "tkind" | 
|     16 and ckind = |     16 and ckind = | 
|     81 | "bv_vs VsNil = []" |     81 | "bv_vs VsNil = []" | 
|     82 | "bv_vs (VsCons v k t) = (atom v) # bv_vs t" |     82 | "bv_vs (VsCons v k t) = (atom v) # bv_vs t" | 
|     83 | "bv_tvs TvsNil = []" |     83 | "bv_tvs TvsNil = []" | 
|     84 | "bv_tvs (TvsCons v k t) = (atom v) # bv_tvs t" |     84 | "bv_tvs (TvsCons v k t) = (atom v) # bv_tvs t" | 
|     85 | "bv_cvs CvsNil = []" |     85 | "bv_cvs CvsNil = []" | 
|     86 | "bv_cvs (CvsCons v k t) = (atom v) # bv_cvs t"     |     86 | "bv_cvs (CvsCons v k t) = (atom v) # bv_cvs t" | 
|     87   |         | 
|     88  |     87  | 
|     89  |     88  | 
|     90 lemmas fv_supp=tkind_ckind_ty_ty_lst_co_co_lst_trm_assoc_lst_pat_vars_tvars_cvars.supp(1-9,11,13,15) |     89 lemmas fv_supp=tkind_ckind_ty_ty_lst_co_co_lst_trm_assoc_lst_pat_vars_tvars_cvars.supp(1-9,11,13,15) | 
|     91 lemmas supp=tkind_ckind_ty_ty_lst_co_co_lst_trm_assoc_lst_pat_vars_tvars_cvars.fv[simplified fv_supp] |     90 lemmas supp=tkind_ckind_ty_ty_lst_co_co_lst_trm_assoc_lst_pat_vars_tvars_cvars.fv[simplified fv_supp] | 
|     92 lemmas perm=tkind_ckind_ty_ty_lst_co_co_lst_trm_assoc_lst_pat_vars_tvars_cvars.perm |     91 lemmas perm=tkind_ckind_ty_ty_lst_co_co_lst_trm_assoc_lst_pat_vars_tvars_cvars.perm |