equal
deleted
inserted
replaced
203 text {* The paper has no Example 10! *} |
203 text {* The paper has no Example 10! *} |
204 |
204 |
205 lemma "(\<forall>A. 0 \<in> A \<and> (\<forall>x \<in> A. Suc x \<in> A) \<longrightarrow> n \<in> A) \<and> |
205 lemma "(\<forall>A. 0 \<in> A \<and> (\<forall>x \<in> A. Suc x \<in> A) \<longrightarrow> n \<in> A) \<and> |
206 P 0 \<and> (\<forall>x. P x \<longrightarrow> P (Suc x)) \<longrightarrow> P n" |
206 P 0 \<and> (\<forall>x. P x \<longrightarrow> P (Suc x)) \<longrightarrow> P n" |
207 -- {* Example 11: needs a hint. *} |
207 -- {* Example 11: needs a hint. *} |
208 by(metis Nat.induct) |
208 by(metis nat.induct) |
209 |
209 |
210 lemma |
210 lemma |
211 "(\<forall>A. (0, 0) \<in> A \<and> (\<forall>x y. (x, y) \<in> A \<longrightarrow> (Suc x, Suc y) \<in> A) \<longrightarrow> (n, m) \<in> A) |
211 "(\<forall>A. (0, 0) \<in> A \<and> (\<forall>x y. (x, y) \<in> A \<longrightarrow> (Suc x, Suc y) \<in> A) \<longrightarrow> (n, m) \<in> A) |
212 \<and> P n \<longrightarrow> P m" |
212 \<and> P n \<longrightarrow> P m" |
213 -- {* Example 12. *} |
213 -- {* Example 12. *} |