Nominal/Ex/CoreHaskell.thy
changeset 2213 231a20534950
parent 2142 c39d4fe31100
child 2312 ad03df7e8056
--- a/Nominal/Ex/CoreHaskell.thy	Sun Jun 06 13:16:27 2010 +0200
+++ b/Nominal/Ex/CoreHaskell.thy	Mon Jun 07 11:33:00 2010 +0200
@@ -84,7 +84,9 @@
 | "bv_tvs TvsNil = []"
 | "bv_tvs (TvsCons v k t) = (atom v) # bv_tvs t"
 | "bv_cvs CvsNil = []"
-| "bv_cvs (CvsCons v k t) = (atom v) # bv_cvs t"    
+| "bv_cvs (CvsCons v k t) = (atom v) # bv_cvs t"
+
+    
 
 lemmas fv_supp=tkind_ckind_ty_ty_lst_co_co_lst_trm_assoc_lst_pat_vars_tvars_cvars.supp(1-9,11,13,15)
 lemmas supp=tkind_ckind_ty_ty_lst_co_co_lst_trm_assoc_lst_pat_vars_tvars_cvars.fv[simplified fv_supp]