# HG changeset patch # User Cezary Kaliszyk # Date 1265111292 -3600 # Node ID 278253330b6ad3b55a7ac3cc9ef8fa14f26fb0a7 # Parent 559419060d99b70fa74bb58db1bb651ccb65a415 Disambiguating the syntax. diff -r 559419060d99 -r 278253330b6a Quot/Nominal/Abs.thy --- a/Quot/Nominal/Abs.thy Tue Feb 02 12:36:01 2010 +0100 +++ b/Quot/Nominal/Abs.thy Tue Feb 02 12:48:12 2010 +0100 @@ -53,7 +53,7 @@ "(alpha_gen (bs, x) R f pi (cs, y)) \ (f x - bs = f y - cs) \ ((f x - bs) \* pi) \ (R (pi \ x) y)" notation - alpha_gen ("_ \gen _ _ _ _") + alpha_gen ("_ \gen _ _ _ _" [100, 100, 100, 100, 100] 100) lemma [mono]: "R1 \ R2 \ alpha_gen x R1 \ alpha_gen x R2" by (cases x) (auto simp add: le_fun_def le_bool_def alpha_gen.simps) @@ -71,7 +71,7 @@ lemma alpha_gen_atom_sym: assumes a: "\pi t s. (R t s \ R (pi \ t) (pi \ s))" - shows "\pi. ({atom a}, t) \gen \x1 x2. R x1 x2 \ R x2 x1 f pi ({atom b}, s) \ + shows "\pi. ({atom a}, t) \gen (\x1 x2. R x1 x2 \ R x2 x1) f pi ({atom b}, s) \ \pi. ({atom b}, s) \gen R f pi ({atom a}, t)" apply(erule exE) apply(rule_tac x="- pi" in exI) @@ -97,7 +97,7 @@ lemma alpha_gen_atom_trans: assumes a: "\pi t s. (R t s \ R (pi \ t) (pi \ s))" - shows "\\pi\perm. ({atom a}, t) \gen \x1 x2. R x1 x2 \ (\x. R x2 x \ R x1 x) f pi ({atom aa}, ta); + shows "\\pi\perm. ({atom a}, t) \gen (\x1 x2. R x1 x2 \ (\x. R x2 x \ R x1 x)) f pi ({atom aa}, ta); \pi\perm. ({atom aa}, ta) \gen R f pi ({atom ba}, sa)\ \ \pi\perm. ({atom a}, t) \gen R f pi ({atom ba}, sa)" apply(simp add: alpha_gen.simps) @@ -131,7 +131,7 @@ lemma alpha_gen_atom_eqvt: assumes a: "\x. pi \ (f x) = f (pi \ x)" - and b: "\pia. ({atom a}, t) \gen \x1 x2. R x1 x2 \ R (pi \ x1) (pi \ x2) f pia ({atom b}, s)" + and b: "\pia. ({atom a}, t) \gen (\x1 x2. R x1 x2 \ R (pi \ x1) (pi \ x2)) f pia ({atom b}, s)" shows "\pia. ({atom (pi \ a)}, pi \ t) \gen R f pia ({atom (pi \ b)}, pi \ s)" using b apply - apply(erule exE) diff -r 559419060d99 -r 278253330b6a Quot/Nominal/LamEx2.thy --- a/Quot/Nominal/LamEx2.thy Tue Feb 02 12:36:01 2010 +0100 +++ b/Quot/Nominal/LamEx2.thy Tue Feb 02 12:48:12 2010 +0100 @@ -371,7 +371,7 @@ lemma alpha_induct: "\qx = qxa; \a b. a = b \ qxb (Var a) (Var b); \x xa xb xc. \x = xa; qxb x xa; xb = xc; qxb xb xc\ \ qxb (App x xb) (App xa xc); - \a t b s. \pi. ({atom a}, t) \gen \x1 x2. x1 = x2 \ qxb x1 x2 fv pi ({atom b}, s) \ qxb (Lam a t) (Lam b s)\ + \a t b s. \pi. ({atom a}, t) \gen (\x1 x2. x1 = x2 \ qxb x1 x2) fv pi ({atom b}, s) \ qxb (Lam a t) (Lam b s)\ \ qxb qx qxa" unfolding alpha_gen by (lifting alpha.induct[unfolded alpha_gen])