# HG changeset patch # User urbanc # Date 1141205268 -3600 # Node ID 0eccb98b1fdbae1ca1c2846d00bd7231ccdd11ca # Parent b61039bf141fc971448269eb45e559ac4b7d6a9b added initialisation-code for finite_guess diff -r b61039bf141f -r 0eccb98b1fdb src/HOL/Nominal/Nominal.thy --- a/src/HOL/Nominal/Nominal.thy Wed Mar 01 10:27:01 2006 +0100 +++ b/src/HOL/Nominal/Nominal.thy Wed Mar 01 10:27:48 2006 +0100 @@ -556,6 +556,13 @@ shows "[(a,b)] \ [(b,a)]" by (force simp add: prm_eq_def at_calc[OF at]) +lemma at_ds5': + fixes a :: "'x" + and b :: "'x" + assumes at: "at TYPE('x)" + shows "[(a,b),(b,a)] \ []" + by (force simp add: prm_eq_def at_calc[OF at]) + lemma at_ds6: fixes a :: "'x" and b :: "'x" @@ -1018,6 +1025,20 @@ shows "[(a,b)]\([(a,b)]\x) = x" by (rule pt_bij2[OF pt, OF at], simp) +lemma pt_swap_bij': + fixes a :: "'x" + and b :: "'x" + and x :: "'a" + assumes pt: "pt TYPE('a) TYPE('x)" + and at: "at TYPE('x)" + shows "[(a,b)]\([(b,a)]\x) = x" +apply(simp add: pt2[OF pt,symmetric]) +apply(rule trans) +apply(rule pt3[OF pt]) +apply(rule at_ds5'[OF at]) +apply(rule pt1[OF pt]) +done + lemma pt_set_bij1: fixes pi :: "'x prm" and x :: "'a" @@ -2747,4 +2768,11 @@ {* supports_meth_debug *} {* tactic for deciding whether something supports something else including debuging facilities *} +method_setup finite_guess = + {* finite_gs_meth *} + {* tactic for deciding whether something has finite support *} + +method_setup finite_guess_debug = + {* finite_gs_meth_debug *} + {* tactic for deciding whether something has finite support including debuging facilities *} end