Nominal/Ex/Ex2.thy
changeset 2309 13f20fe02ff3
parent 2301 8732ff59068b
child 2311 4da5c5c29009
--- a/Nominal/Ex/Ex2.thy	Wed Jun 02 11:37:51 2010 +0200
+++ b/Nominal/Ex/Ex2.thy	Thu Jun 03 11:48:44 2010 +0200
@@ -3,7 +3,7 @@
 begin
 
 text {* example 2 *}
-declare [[STEPS = 8]]
+declare [[STEPS = 9]]
 
 atom_decl name
 
@@ -23,6 +23,7 @@
 | "f (PD x y) = {atom x, atom y}"
 | "f (PS x) = {atom x}"
 
+
 thm fv_trm_raw.simps[no_vars] fv_pat_raw.simps[no_vars] fv_f_raw.simps[no_vars] f_raw.simps[no_vars]
 thm alpha_trm_raw_alpha_pat_raw_alpha_f_raw.intros[no_vars]