doc-src/TutorialI/Overview/Ind.thy
changeset 11293 6878bb02a7f9
parent 11235 860c65c7388a
child 12815 1f073030b97a
--- a/doc-src/TutorialI/Overview/Ind.thy	Thu May 10 09:41:45 2001 +0200
+++ b/doc-src/TutorialI/Overview/Ind.thy	Thu May 10 09:48:50 2001 +0200
@@ -88,8 +88,16 @@
   acc :: "('a \<times> 'a) set \<Rightarrow> 'a set"
 inductive "acc r"
 intros
-  "(\<forall>y. (x,y) \<in> r \<longrightarrow> y \<in> acc r) \<Longrightarrow> x \<in> acc r"
+  "(\<forall>y. (y,x) \<in> r \<longrightarrow> y \<in> acc r) \<Longrightarrow> x \<in> acc r"
 
+lemma "wf{(x,y). (x,y) \<in> r \<and> y \<in> acc r}"
+thm wfI
+apply(rule_tac A = "acc r" in wfI)
+ apply (blast elim:acc.elims)
+apply(simp(no_asm_use))
+thm acc.induct
+apply(erule acc.induct)
+by blast
 
 consts
   accs :: "('a \<times> 'a) set \<Rightarrow> 'a set"