Static.thy
changeset 74 271e9818b6f6
parent 67 811e3028d169
--- a/Static.thy	Wed Nov 20 21:33:56 2013 +0800
+++ b/Static.thy	Mon Dec 02 10:52:40 2013 +0800
@@ -359,7 +359,7 @@
      (\<forall> sec flag sf'. (sec,flag,sf') \<in> sfds \<and> (sf \<preceq> sf') \<longrightarrow> 
          (sec, flag, sf') \<in> sfds' \<and> (sec,flag, file_after_rename sf' from to) \<notin> sfds')"
 
-(* for not many, choose on renamed or not *)
+  (* for not many, choose on renamed or not *)
 definition sfds_rename_choices
   :: "t_sfd set \<Rightarrow> t_sfile \<Rightarrow> t_sfile \<Rightarrow> t_sfile \<Rightarrow> t_sfd set \<Rightarrow> bool"
 where