diff -r 216e31270509 -r 843da46f89ac src/HOL/Unix/Unix.thy --- a/src/HOL/Unix/Unix.thy Sat Jan 21 23:02:20 2006 +0100 +++ b/src/HOL/Unix/Unix.thy Sat Jan 21 23:02:21 2006 +0100 @@ -653,11 +653,11 @@ "can_exec root xs \ \root'. root =xs\ root'" lemma can_exec_nil: "can_exec root []" - by (unfold can_exec_def) (blast intro: transitions.intros) + unfolding can_exec_def by (blast intro: transitions.intros) lemma can_exec_cons: "root \x\ root' \ can_exec root' xs \ can_exec root (x # xs)" - by (unfold can_exec_def) (blast intro: transitions.intros) + unfolding can_exec_def by (blast intro: transitions.intros) text {* \medskip In case that we already know that a certain sequence can be @@ -677,7 +677,7 @@ xs_y: "r =(xs @ [y])\ root''" by (auto simp add: can_exec_def transitions_nil_eq transitions_cons_eq) from xs_y Cons.hyps obtain root' r' where xs: "r =xs\ root'" and y: "root' \y\ r'" - by (unfold can_exec_def) blast + unfolding can_exec_def by blast from x xs have "root =(x # xs)\ root'" by (rule transitions.cons) with y show ?case by blast @@ -913,7 +913,7 @@ shows False proof - from inv obtain "file" where "access root bogus_path user\<^isub>1 {} = Some file" - by (unfold invariant_def) blast + unfolding invariant_def by blast moreover from rmdir obtain att where "access root [user\<^isub>1, name\<^isub>1] user\<^isub>1 {} = Some (Env att empty)" @@ -1076,7 +1076,7 @@ from inv3 lookup' and not_writable user\<^isub>1_not_root have "access root' path user\<^isub>1 {Writable} = None" by (simp add: access_def) - with inv1' inv2' inv3 show ?thesis by (unfold invariant_def) blast + with inv1' inv2' inv3 show ?thesis unfolding invariant_def by blast qed qed qed