doc-src/TutorialI/Inductive/AB.thy
changeset 11870 181bd2050cf4
parent 11705 ac8ca15c556c
child 12332 aea72a834c85
--- a/doc-src/TutorialI/Inductive/AB.thy	Mon Oct 22 11:55:35 2001 +0200
+++ b/doc-src/TutorialI/Inductive/AB.thy	Mon Oct 22 12:01:35 2001 +0200
@@ -117,7 +117,7 @@
 
 lemma step1: "\<forall>i < size w.
   \<bar>(int(size[x\<in>take (i+1) w. P x])-int(size[x\<in>take (i+1) w. \<not>P x]))
-   - (int(size[x\<in>take i w. P x])-int(size[x\<in>take i w. \<not>P x]))\<bar> \<le> Numeral1"
+   - (int(size[x\<in>take i w. P x])-int(size[x\<in>take i w. \<not>P x]))\<bar> \<le> 1"
 
 txt{*\noindent
 The lemma is a bit hard to read because of the coercion function
@@ -150,7 +150,7 @@
 @{thm[source]step1}:
 *}
 
-apply(insert nat0_intermed_int_val[OF step1, of "P" "w" "Numeral1"])
+apply(insert nat0_intermed_int_val[OF step1, of "P" "w" "1"])
 by force
 
 text{*\noindent