Nominal/Ex/FiniteType.thy
branchNominal2-Isabelle2012
changeset 3170 89715c48f728
parent 3169 b6873d123f9b
child 3171 f5057aabf5c0
--- a/Nominal/Ex/FiniteType.thy	Sat May 12 21:39:09 2012 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,19 +0,0 @@
-theory FiniteType
-imports "../Nominal2"
-begin
-
-typedef ('a::pt, 'b::fs) ffun = "{f::'a => 'b. finite (supp f)}"
-apply(rule_tac x="\<lambda>_. undefined::'b::fs" in exI)
-apply(auto)
-apply(rule_tac S="supp (undefined::'b::fs)" in supports_finite)
-apply(simp add: supports_def)
-apply(perm_simp)
-apply(simp add: fresh_def[symmetric])
-apply(simp add: swap_fresh_fresh)
-apply(simp add: finite_supp)
-done
-
-
-
-
-end
\ No newline at end of file