diff -r 23a8c5ac35f8 -r 69916a850301 src/HOL/Bali/TypeRel.thy --- a/src/HOL/Bali/TypeRel.thy Sat Oct 17 01:05:59 2009 +0200 +++ b/src/HOL/Bali/TypeRel.thy Sat Oct 17 14:43:18 2009 +0200 @@ -59,12 +59,12 @@ translations - "G\I \I1 J" == "(I,J) \ subint1 G" - "G\I \I J" == "(I,J) \(subint1 G)^*" --{* cf. 9.1.3 *} - (* Defined in Decl.thy: + "G\I \I1 J" == "(I,J) \ subint1 G" + "G\I \I J" == "(I,J) \(subint1 G)^*" --{* cf. 9.1.3 *} + (* Defined in Decl.thy: "G\C \\<^sub>C\<^sub>1 D" == "(C,D) \ subcls1 G" - "G\C \\<^sub>C D" == "(C,D) \(subcls1 G)^*" - *) + "G\C \\<^sub>C D" == "(C,D) \(subcls1 G)^*" + *) "G\C \1 I" == "(C,I) \ implmt1 G" @@ -202,12 +202,12 @@ assume subcls_D_C: "G\D \\<^sub>C C" show "False" proof - - from subcls_D_C subcls1_C_Z - have "G\D \\<^sub>C Z" - by (auto dest: r_into_trancl trancl_trans) - with nsubcls_D_Z - show ?thesis - by (rule notE) + from subcls_D_C subcls1_C_Z + have "G\D \\<^sub>C Z" + by (auto dest: r_into_trancl trancl_trans) + with nsubcls_D_Z + show ?thesis + by (rule notE) qed qed qed @@ -243,16 +243,16 @@ assume eq_C_D: "C=D" show "False" proof - - from subcls1_C_Z eq_C_D - have "G\D \\<^sub>C Z" - by (auto) - also - from subcls_Z_D ws - have "\ G\D \\<^sub>C Z" - by (rule subcls_acyclic) - ultimately - show ?thesis - by - (rule notE) + from subcls1_C_Z eq_C_D + have "G\D \\<^sub>C Z" + by (auto) + also + from subcls_Z_D ws + have "\ G\D \\<^sub>C Z" + by (rule subcls_acyclic) + ultimately + show ?thesis + by - (rule notE) qed qed qed @@ -298,12 +298,12 @@ case Eq with ws subcls_C_D show ?thesis - by (auto dest: subcls_irrefl) + by (auto dest: subcls_irrefl) next case Subcls with nsubcls_D_C show ?thesis - by blast + by blast qed qed qed @@ -387,7 +387,7 @@ inductive --{*widening, viz. method invocation conversion, cf. 5.3 - i.e. kind of syntactic subtyping *} + i.e. kind of syntactic subtyping *} widen :: "prog \ ty \ ty \ bool" ("_\_\_" [71,71,71] 70) for G :: prog where @@ -619,8 +619,8 @@ | obj_arr: "G\Class Object\T.[]" | int_cls: "G\ Iface I\Class C" | subint: "imethds G I hidings imethds G J entails - (\(md, mh ) (md',mh').\G\mrt mh\mrt mh') \ - \G\I\I J \\\\ G\ Iface I\Iface J" + (\(md, mh ) (md',mh').\G\mrt mh\mrt mh') \ + \G\I\I J \\\\ G\ Iface I\Iface J" | array: "G\RefT S\RefT T \\ G\ RefT S.[]\RefT T.[]" (*unused*) @@ -637,7 +637,7 @@ by (ind_cases "G\PrimT pt\T") lemma narrow_PrimT2: "G\S\PrimT pt \ - \t. S=PrimT t \ G\PrimT t\PrimT pt" + \t. S=PrimT t \ G\PrimT t\PrimT pt" by (ind_cases "G\S\PrimT pt") text {*