equal
deleted
inserted
replaced
589 |
589 |
590 theorem transitions_type_safe: |
590 theorem transitions_type_safe: |
591 assumes "root =xs\<Rightarrow> root'" |
591 assumes "root =xs\<Rightarrow> root'" |
592 and "\<exists>att dir. root = Env att dir" |
592 and "\<exists>att dir. root = Env att dir" |
593 shows "\<exists>att dir. root' = Env att dir" |
593 shows "\<exists>att dir. root' = Env att dir" |
594 using transition_type_safe and prems |
594 using transition_type_safe and assms |
595 proof (rule transitions_invariant) |
595 proof (rule transitions_invariant) |
596 show "\<forall>x \<in> set xs. True" by blast |
596 show "\<forall>x \<in> set xs. True" by blast |
597 qed |
597 qed |
598 |
598 |
599 |
599 |