# HG changeset patch # User urbanc # Date 1315419409 0 # Node ID 161128ccb65a1095e32744af91604a019ebd9a3c # Parent 40b8d485ce8d85099386f2127a63447a9dfc379c typos diff -r 40b8d485ce8d -r 161128ccb65a Derivatives.thy --- a/Derivatives.thy Wed Sep 07 09:28:13 2011 +0000 +++ b/Derivatives.thy Wed Sep 07 18:16:49 2011 +0000 @@ -115,7 +115,7 @@ by (induct s arbitrary: r) (simp_all add: Deriv_deriv) -subsection {* Antimirov's partial derivivatives *} +subsection {* Antimirov's partial derivatives *} abbreviation "Timess rs r \ {Times r' r | r'. r' \ rs}" @@ -165,7 +165,7 @@ shows "pderivs s (Atom c) \ {Atom c, One}" by (induct s) (simp_all) -subsection {* Relating left-quotients and partial derivivatives *} +subsection {* Relating left-quotients and partial derivatives *} lemma Deriv_pderiv: shows "Deriv c (lang r) = \ lang ` (pderiv c r)" @@ -186,7 +186,7 @@ finally show "Derivs (c # s) (lang r) = \ lang ` pderivs (c # s) r" . qed (simp add: Derivs_def) -subsection {* Relating derivivatives and partial derivivatives *} +subsection {* Relating derivatives and partial derivatives *} lemma deriv_pderiv: shows "(\ lang ` (pderiv c r)) = lang (deriv c r)" @@ -197,7 +197,7 @@ unfolding Derivs_derivs[symmetric] Derivs_pderivs by simp -subsection {* Finiteness property of partial derivivatives *} +subsection {* Finiteness property of partial derivatives *} definition pderivs_lang :: "'a lang \ 'a rexp \ 'a rexp set" @@ -244,7 +244,7 @@ unfolding UNIV1_def pderivs_lang_def by auto -text {* Non-empty suffixes of a string (needed for teh cases of @{const Times} and @{const Star} *} +text {* Non-empty suffixes of a string (needed for the cases of @{const Times} and @{const Star} below) *} definition "PSuf s \ {v. v \ [] \ (\u. u @ v = s)}"