Added lemma at_fin_set_fresh.
authorberghofe
Thu, 24 Jan 2008 11:23:11 +0100
changeset 25950 a3067f6f08a2
parent 25949 850b4c2d0f17
child 25951 6ebe26bfed18
Added lemma at_fin_set_fresh.
src/HOL/Nominal/Nominal.thy
--- a/src/HOL/Nominal/Nominal.thy	Wed Jan 23 23:35:23 2008 +0100
+++ b/src/HOL/Nominal/Nominal.thy	Thu Jan 24 11:23:11 2008 +0100
@@ -1947,6 +1947,13 @@
   then show "X\<subseteq>(supp X)" by blast
 qed
 
+lemma at_fin_set_fresh:
+  fixes X::"'x set" 
+  assumes at: "at TYPE('x)"
+  and     fs: "finite X"
+  shows "(x \<sharp> X) = (x \<notin> X)"
+  by (simp add: at_fin_set_supp fresh_def at fs)
+
 section {* Permutations acting on Functions *}
 (*==========================================*)