# HG changeset patch # User wenzelm # Date 973283662 -3600 # Node ID ac1ae85a56051dd7fe65f80e023c9a11bdd6b9dd # Parent 9dac2cad550097d381c7572ae69fcb0c9a3d7edc tuned notation; diff -r 9dac2cad5500 -r ac1ae85a5605 src/HOL/Library/Accessible_Part.thy --- a/src/HOL/Library/Accessible_Part.thy Fri Nov 03 21:33:53 2000 +0100 +++ b/src/HOL/Library/Accessible_Part.thy Fri Nov 03 21:34:22 2000 +0100 @@ -28,7 +28,7 @@ syntax termi :: "('a \ 'a) set => 'a set" translations - "termi r" == "acc (r^-1)" + "termi r" == "acc (r\)" subsection {* Induction rules *} @@ -53,13 +53,13 @@ apply fast done -lemma acc_downwards_aux: "(b, a) \ r^* ==> a \ acc r --> b \ acc r" +lemma acc_downwards_aux: "(b, a) \ r\<^sup>* ==> a \ acc r --> b \ acc r" apply (erule rtrancl_induct) apply blast apply (blast dest: acc_downward) done -theorem acc_downwards: "a \ acc r ==> (b, a) \ r^* ==> b \ acc r" +theorem acc_downwards: "a \ acc r ==> (b, a) \ r\<^sup>* ==> b \ acc r" apply (blast dest: acc_downwards_aux) done