src/HOL/Induct/Acc.thy
changeset 7721 cb353d802ade
parent 5717 0d28dbe484b6
child 7759 44dd5dc8e90f
--- a/src/HOL/Induct/Acc.thy	Tue Oct 05 15:31:39 1999 +0200
+++ b/src/HOL/Induct/Acc.thy	Tue Oct 05 15:31:42 1999 +0200
@@ -9,19 +9,15 @@
 Research Report 92-49, LIP, ENS Lyon.  Dec 1992.
 *)
 
-Acc = WF + Inductive +
-
-constdefs
-  pred :: "['b, ('a * 'b)set] => 'a set"        (*Set of predecessors*)
-  "pred x r == {y. (y,x):r}"
+theory Acc = WF + Inductive:
 
 consts
   acc  :: "('a * 'a)set => 'a set"              (*Accessible part*)
 
-inductive "acc(r)"
+inductive "acc r"
   intrs
-    pred    "pred a r: Pow(acc(r)) ==> a: acc(r)"
-  monos     Pow_mono
+    accI [rulify_prems]: "ALL y. (y, x) : r --> y : acc r ==> x : acc r"
+
 
 syntax        termi :: "('a * 'a)set => 'a set"
 translations "termi r" == "acc(r^-1)"