src/HOL/MicroJava/Comp/Index.thy
changeset 17778 93d7e524417a
parent 16417 9bc16273c2d4
child 27117 97e9dae57284
--- a/src/HOL/MicroJava/Comp/Index.thy	Fri Oct 07 18:49:20 2005 +0200
+++ b/src/HOL/MicroJava/Comp/Index.thy	Fri Oct 07 20:41:10 2005 +0200
@@ -5,7 +5,9 @@
 
 (* Index of variable in list of parameter names and local variables *)
 
-theory Index imports  AuxLemmas DefsComp begin
+theory Index
+imports AuxLemmas DefsComp
+begin
 
 (*indexing a variable name among all variable declarations in a method body*)
 constdefs
@@ -76,7 +78,6 @@
 apply (case_tac b, simp)
 apply (rule conjI)
 apply (simp add: gl_def)
-apply (intro strip, simp)
 apply (simp add: galldefs del: set_append map_append)
 done