src/HOL/MicroJava/J/Conform.thy
changeset 12888 f6c1e7306c40
parent 12517 360e3215f029
child 12911 704713ca07ea
--- a/src/HOL/MicroJava/J/Conform.thy	Thu Feb 14 11:50:52 2002 +0100
+++ b/src/HOL/MicroJava/J/Conform.thy	Thu Feb 14 12:06:07 2002 +0100
@@ -238,7 +238,7 @@
 done
 
 lemma lconf_ext_list [rule_format (no_asm)]: 
-  "G,h\<turnstile>l[::\<preceq>]L ==> \<forall>vs Ts. nodups vns --> length Ts = length vns --> 
+  "G,h\<turnstile>l[::\<preceq>]L ==> \<forall>vs Ts. distinct vns --> length Ts = length vns --> 
   list_all2 (\<lambda>v T. G,h\<turnstile>v::\<preceq>T) vs Ts --> G,h\<turnstile>l(vns[\<mapsto>]vs)[::\<preceq>]L(vns[\<mapsto>]Ts)"
 apply (unfold lconf_def)
 apply( induct_tac "vns")