equal
deleted
inserted
replaced
768 finally show ?thesis . |
768 finally show ?thesis . |
769 qed |
769 qed |
770 thus ?thesis by (simp add:restm_def) |
770 thus ?thesis by (simp add:restm_def) |
771 qed |
771 qed |
772 |
772 |
|
773 lemma moment_prefix: "(moment i t @ s) = moment (i + length s) (t @ s)" |
|
774 proof - |
|
775 from moment_plus_split [of i "length s" "t@s"] |
|
776 have " moment (i + length s) (t @ s) = moment i (restm (length s) (t @ s)) @ moment (length s) (t @ s)" |
|
777 by auto |
|
778 with app_moment_restm[of t s] |
|
779 have "moment (i + length s) (t @ s) = moment i t @ moment (length s) (t @ s)" by simp |
|
780 with moment_app show ?thesis by auto |
|
781 qed |
|
782 |
773 end |
783 end |