Theory More_Sublist
section ‹Lemmas on sublists›
theory More_Sublist
imports
"HOL-Library.Sublist"
begin
lemma same_length_is_parallel:
assumes len: "∀y ∈ set as. length y = x"
shows "∀x ∈ set as. ∀y ∈ set as - {x}. x ∥ y"
proof (rule, rule)
fix x y
assume xi: "x ∈ set as" and yi: "y ∈ set as - {x}"
from len obtain q where len': "∀y ∈ set as. length y = q" ..
show "x ∥ y"
proof (rule not_equal_is_parallel)
from xi yi show "x ≠ y" by auto
from xi yi len' show "length x = length y" by (auto dest: bspec)
qed
qed
lemma sublist_equal_part:
"prefix xs ys ⟹ take (length xs) ys = xs"
by (clarsimp simp: prefix_def)
lemma prefix_length_less:
"strict_prefix xs ys ⟹ length xs < length ys"
apply (clarsimp simp: strict_prefix_def)
apply (frule prefix_length_le)
apply (rule ccontr, simp)
apply (clarsimp simp: prefix_def)
done
lemmas take_less = take_strict_prefix
lemma not_prefix_longer:
"⟦ length xs > length ys ⟧ ⟹ ¬ prefix xs ys"
by (clarsimp dest!: prefix_length_le)
lemma map_prefixI:
"prefix xs ys ⟹ prefix (map f xs) (map f ys)"
by (clarsimp simp: prefix_def)
lemma list_all2_induct_suffixeq [consumes 1, case_names Nil Cons]:
assumes lall: "list_all2 Q as bs"
and nilr: "P [] []"
and consr: "⋀x xs y ys.
⟦list_all2 Q xs ys; Q x y; P xs ys; suffix (x # xs) as; suffix (y # ys) bs⟧
⟹ P (x # xs) (y # ys)"
shows "P as bs"
proof -
define as' where "as' == as"
define bs' where "bs' == bs"
have "suffix as as' ∧ suffix bs bs'" unfolding as'_def bs'_def by simp
then show ?thesis using lall
proof (induct rule: list_induct2 [OF list_all2_lengthD [OF lall]])
case 1 show ?case by fact
next
case (2 x xs y ys)
show ?case
proof (rule consr)
from "2.prems" show "list_all2 Q xs ys" and "Q x y" by simp_all
then show "P xs ys" using "2.hyps" "2.prems" by (auto dest: suffix_ConsD)
from "2.prems" show "suffix (x # xs) as" and "suffix (y # ys) bs"
by (auto simp: as'_def bs'_def)
qed
qed
qed
lemma take_prefix:
"(take (length xs) ys = xs) = prefix xs ys"
proof (induct xs arbitrary: ys)
case Nil then show ?case by simp
next
case Cons then show ?case by (cases ys) auto
qed
end