diff -r f63bca3e574e -r 85fb973a8207 src/HOL/Nominal/Examples/Crary.thy --- a/src/HOL/Nominal/Examples/Crary.thy Sun Aug 12 14:14:24 2007 +0200 +++ b/src/HOL/Nominal/Examples/Crary.thy Sun Aug 12 18:53:03 2007 +0200 @@ -274,6 +274,7 @@ "\\<^isub>1 \ \\<^isub>2 \ \a T. (a,T)\set \\<^isub>1 \ (a,T)\set \\<^isub>2" lemma valid_monotonicity[elim]: + fixes \ \' :: Ctxt assumes a: "\ \ \'" and b: "x\\'" shows "(x,T\<^isub>1)#\ \ (x,T\<^isub>1)#\'" @@ -373,6 +374,7 @@ done lemma test3a: + fixes \ :: Ctxt and t :: trm assumes a: "\ \ t : T" shows "(supp t) \ ((supp \)::name set)" using a @@ -392,6 +394,7 @@ done lemma test3: + fixes \ :: Ctxt and s t :: trm assumes a: "\ \ s \ t : T" shows "(supp (s,t)) \ ((supp \)::name set)" using a @@ -765,7 +768,8 @@ apply(auto) done -lemma logical_monotonicity : +lemma logical_monotonicity: + fixes \ \' :: Ctxt assumes a1: "\ \ s is t : T" and a2: "\ \ \'" and a3: "valid \'" @@ -915,6 +919,7 @@ qed lemma logical_subst_monotonicity : + fixes \ \' \'' :: Ctxt assumes a: "\' \ \ is \' over \" and b: "\' \ \''" and c: "valid \''"