| changeset 12566 | fe20540bcf93 |
| parent 12517 | 360e3215f029 |
| child 12911 | 704713ca07ea |
--- a/src/HOL/MicroJava/J/WellForm.thy Thu Dec 20 17:08:55 2001 +0100 +++ b/src/HOL/MicroJava/J/WellForm.thy Thu Dec 20 18:22:44 2001 +0100 @@ -178,7 +178,7 @@ apply( assumption) apply( fast) apply(auto dest!: wf_cdecl_supD) -apply(erule (1) rtrancl_into_rtrancl2) +apply(erule (1) converse_rtrancl_into_rtrancl) done lemma is_type_rTI: "wf_mhead G sig rT ==> is_type G rT"