Experiments with equivariance.
authorCezary Kaliszyk <kaliszyk@in.tum.de>
Thu, 06 May 2010 10:43:41 +0200
changeset 2067 ace7775cbd04
parent 2066 deb732753522
child 2068 79b733010bc5
Experiments with equivariance.
Nominal/Ex/Ex1rec.thy
Nominal/Ex/ExLetRec.thy
--- a/Nominal/Ex/Ex1rec.thy	Wed May 05 20:39:56 2010 +0100
+++ b/Nominal/Ex/Ex1rec.thy	Thu May 06 10:43:41 2010 +0200
@@ -29,6 +29,11 @@
 ML {* Sign.of_sort @{theory} (@{typ lam}, @{sort fs}) *}
 thm lam_bp.fv[simplified lam_bp.supp(1-2)]
 
+(*declare permute_lam_raw_permute_bp_raw.simps[eqvt]
+declare alpha_gen_eqvt[eqvt]
+equivariance alpha_lam_raw
+*)
+
 end
 
 
--- a/Nominal/Ex/ExLetRec.thy	Wed May 05 20:39:56 2010 +0100
+++ b/Nominal/Ex/ExLetRec.thy	Thu May 06 10:43:41 2010 +0200
@@ -75,6 +75,12 @@
   apply (simp add: atom_eqvt fresh_star_def)
   done
 
+(*
+declare permute_trm_raw_permute_lts_raw.simps[eqvt]
+declare alpha_gen_eqvt[eqvt]
+equivariance alpha_trm_raw
+*)
+
 end