src/HOL/Bali/WellForm.thy
changeset 37678 0040bafffdef
parent 35440 bdf8ad377877
child 37956 ee939247b2fb
--- a/src/HOL/Bali/WellForm.thy	Thu Jul 01 16:54:42 2010 +0200
+++ b/src/HOL/Bali/WellForm.thy	Thu Jul 01 16:54:44 2010 +0200
@@ -2168,7 +2168,7 @@
       by (force dest!: ws_dynmethd accmethd_SomeD)
     with dynlookup eq_mheads 
     show ?thesis 
-      by (cases emh type: *) (auto)
+      by (cases emh type: prod) (auto)
   next
     case Iface_methd
     fix I im
@@ -2191,7 +2191,7 @@
       by (force dest: implmt_methd)
     with dynlookup eq_mheads
     show ?thesis 
-      by (cases emh type: *) (auto)
+      by (cases emh type: prod) (auto)
   next
     case Iface_Object_methd
     fix I sm
@@ -2217,7 +2217,7 @@
                   intro: class_Object [OF wf] intro: that)
        with dynlookup eq_mheads
        show ?thesis 
-         by (cases emh type: *) (auto)
+         by (cases emh type: prod) (auto)
      next
        case False
        with statI
@@ -2243,7 +2243,7 @@
          by (auto dest: implmt_methd)
        with wf eq_stat resProp dynlookup eq_mheads
        show ?thesis 
-         by (cases emh type: *) (auto intro: widen_trans)
+         by (cases emh type: prod) (auto intro: widen_trans)
      qed
   next
     case Array_Object_methd
@@ -2256,7 +2256,7 @@
       by (auto simp add: dynlookup_def dynmethd_C_C)
     with sm eq_mheads sm 
     show ?thesis 
-      by (cases emh type: *) (auto dest: accmethd_SomeD)
+      by (cases emh type: prod) (auto dest: accmethd_SomeD)
   qed
 qed
 declare split_paired_All [simp] split_paired_Ex [simp]