src/HOL/MicroJava/J/Eval.thy
changeset 56073 29e308b56d23
parent 47632 50f9f699b2d7
child 58886 8a6cac7c7247
equal deleted inserted replaced
56072:31e427387ab5 56073:29e308b56d23
   224   proof(cases (no_simp))
   224   proof(cases (no_simp))
   225     case LAcc with LAcc_code show ?thesis by auto
   225     case LAcc with LAcc_code show ?thesis by auto
   226   next
   226   next
   227     case (Call a b c d e f g h i j k l m n o p q r s t u v s4)
   227     case (Call a b c d e f g h i j k l m n o p q r s t u v s4)
   228     with Call_code show ?thesis
   228     with Call_code show ?thesis
   229       by(cases "s4")(simp, (erule meta_allE meta_impE|rule conjI refl| assumption)+)
   229       by(cases "s4") auto
   230   qed(erule (3) that[OF refl]|assumption)+
   230   qed(erule (3) that[OF refl]|assumption)+
   231 next
   231 next
   232   case evals
   232   case evals
   233   from evals.prems show thesis
   233   from evals.prems show thesis
   234     by(cases (no_simp))(erule (3) that[OF refl]|assumption)+
   234     by(cases (no_simp))(erule (3) that[OF refl]|assumption)+