src/HOL/Unix/Unix.thy
changeset 10979 3da4543034e7
parent 10966 8f2c27041a8e
child 11004 af8008e4de96
equal deleted inserted replaced
10978:5eebea8f359f 10979:3da4543034e7
  1062         assume "ys = []"
  1062         assume "ys = []"
  1063         with path have parent: "path_of x = path @ [y]" by simp
  1063         with path have parent: "path_of x = path @ [y]" by simp
  1064         with tr uid inv4 changed obtain file where
  1064         with tr uid inv4 changed obtain file where
  1065             "root' = update (path_of x) (Some file) root"
  1065             "root' = update (path_of x) (Some file) root"
  1066           by cases auto
  1066           by cases auto
  1067         with parent lookup have "lookup root' path = Some (Env att (dir(y\<mapsto>file)))"
  1067         with lookup parent have "lookup root' path = Some (Env att (dir(y\<mapsto>file)))"
  1068           by (simp only: update_append_some update_cons_nil_env)
  1068           by (simp only: update_append_some update_cons_nil_env)
  1069         moreover have "dir(y\<mapsto>file) \<noteq> empty" by simp
  1069         moreover have "dir(y\<mapsto>file) \<noteq> empty" by simp
  1070         ultimately show ?thesis ..
  1070         ultimately show ?thesis ..
  1071       next
  1071       next
  1072         fix z zs assume ys: "ys = z # zs"
  1072         fix z zs assume ys: "ys = z # zs"