src/HOL/Hyperreal/MacLaurin.thy
changeset 15944 9b00875e21f7
parent 15561 045a07ac35a7
child 16775 c1b87ef4a1c3
--- a/src/HOL/Hyperreal/MacLaurin.thy	Mon May 09 16:02:45 2005 +0200
+++ b/src/HOL/Hyperreal/MacLaurin.thy	Mon May 09 16:38:56 2005 +0200
@@ -1,10 +1,11 @@
-(*  Title       : MacLaurin.thy
+(*  ID          : $Id$
     Author      : Jacques D. Fleuriot
     Copyright   : 2001 University of Edinburgh
-    Description : MacLaurin series
     Conversion to Isar and new proofs by Lawrence C Paulson, 2004
 *)
 
+header{*MacLaurin Series*}
+
 theory MacLaurin
 imports Log
 begin
@@ -583,7 +584,7 @@
       in Maclaurin_all_le_objl)
     apply safe
     apply simp
-    apply (simplesubst mod_Suc_eq_Suc_mod)  --{*simultaneous substitution*}
+    apply (subst (1 2 3) mod_Suc_eq_Suc_mod)
     apply (cut_tac m=m in mod_exhaust_less_4, safe, simp+)
     apply (rule DERIV_minus, simp+)
     apply (rule lemma_DERIV_subst, rule DERIV_minus, rule DERIV_cos, simp)