Removed sorry's.

This commit is contained in:
Achim D. Brucker 2016-12-27 10:50:50 +00:00
parent f290da191d
commit 2f0da5f6ba
1 changed files with 0 additions and 2 deletions

View File

@ -609,8 +609,6 @@ lemma rule_charn2:
case Nil show ?case using Nil by simp
next
case (snoc y ys)
then have * : " y = AllowPortFromTo c d po \<Longrightarrow> ys \<noteq> []" sorry
have ** : "applied_rule_rev C x ys = Some (AllowPortFromTo c d po)" sledgehammer sorry
show ?case using snoc
apply (case_tac "y = (AllowPortFromTo c d po)", simp_all )
apply (simp add: applied_rule_rev_def)