diff -r e623e57b0f44 -r 67e9b86ed211 src/HOL/Unix/Unix.thy --- a/src/HOL/Unix/Unix.thy Thu Aug 25 16:13:09 2005 +0200 +++ b/src/HOL/Unix/Unix.thy Thu Aug 25 16:17:40 2005 +0200 @@ -129,7 +129,7 @@ *} types - file = "(att \ string, att, name) env" + "file" = "(att \ string, att, name) env" text {* \medskip The HOL library also provides @{term lookup} and @{term @@ -151,7 +151,7 @@ \cite{Bauer-et-al:2002:HOL-Library}. These will be routinely used later on without further notice. - \bigskip Apparently, the elements of type @{typ file} contain an + \bigskip Apparently, the elements of type @{typ "file"} contain an @{typ att} component in either case. We now define a few auxiliary operations to manipulate this field uniformly, following the conventions for record types in Isabelle/HOL @@ -178,7 +178,7 @@ by (simp add: attributes_def) lemma [simp]: "attributes (file \attributes := att\) = att" - by (cases file) (simp_all add: attributes_def attributes_update_def + by (cases "file") (simp_all add: attributes_def attributes_update_def split_tupled_all) lemma [simp]: "(Val (att, text)) \attributes := att'\ = Val (att', text)" @@ -934,7 +934,7 @@ root \(Rmdir user1 [user1, name1])\ root' \ False" proof - assume "invariant root bogus_path" - then obtain file where "access root bogus_path user1 {} = Some file" + then obtain "file" where "access root bogus_path user1 {} = Some file" by (unfold invariant_def) blast moreover assume "root \(Rmdir user1 [user1, name1])\ root'" @@ -1055,7 +1055,7 @@ proof (cases ys) assume "ys = []" with path have parent: "path_of x = path @ [y]" by simp - with tr uid inv4 changed obtain file where + with tr uid inv4 changed obtain "file" where "root' = update (path_of x) (Some file) root" by cases auto with lookup parent have "lookup root' path = Some (Env att (dir(y\file)))"