Static.thy
changeset 43 137358bd4921
parent 42 021672ec28f5
child 47 0960686df575
--- a/Static.thy	Thu Sep 05 13:23:03 2013 +0800
+++ b/Static.thy	Thu Sep 12 13:50:22 2013 +0800
@@ -172,7 +172,6 @@
 | "is_many (S_dir  sf      ) = is_many_sfile sf"
 | "is_many (S_msgq sq      ) = is_many_smsgq sq"
 | "is_many (S_shm  sh      ) = is_many_sshm  sh"
-| "is_many _                 = False"
 
 (*
 fun update_ss_sp:: "t_static_state \<Rightarrow> t_sobject \<Rightarrow> t_sobject \<Rightarrow> t_static_state"