src/HOL/List.thy
changeset 14327 9cd4dea593e3
parent 14316 91b897b9a2dc
child 14328 fd063037fdf5
equal deleted inserted replaced
14326:c817dd885a32 14327:9cd4dea593e3
  1167   apply (induct as, simp)
  1167   apply (induct as, simp)
  1168   apply (clarsimp simp add: list_all2_Cons1)
  1168   apply (clarsimp simp add: list_all2_Cons1)
  1169   apply (case_tac n, simp, simp)
  1169   apply (case_tac n, simp, simp)
  1170   done
  1170   done
  1171 
  1171 
  1172 lemma list_all2_mono [trans, intro?]:
  1172 lemma list_all2_mono [intro?]:
  1173   "\<And>y. list_all2 P x y \<Longrightarrow> (\<And>x y. P x y \<Longrightarrow> Q x y) \<Longrightarrow> list_all2 Q x y"
  1173   "\<And>y. list_all2 P x y \<Longrightarrow> (\<And>x y. P x y \<Longrightarrow> Q x y) \<Longrightarrow> list_all2 Q x y"
  1174   apply (induct x, simp)
  1174   apply (induct x, simp)
  1175   apply (case_tac y, auto)
  1175   apply (case_tac y, auto)
  1176   done
  1176   done
  1177 
  1177