src/HOL/MicroJava/BV/Correct.thy
changeset 35355 613e133966ea
parent 33954 1bc3b688548c
child 35417 47ee18b6ae32
equal deleted inserted replaced
35354:2e8dc3c64430 35355:613e133966ea
    64        correct_frame G hp s maxl ins f \<and> 
    64        correct_frame G hp s maxl ins f \<and> 
    65              correct_frames G hp phi rT sig fs))
    65              correct_frames G hp phi rT sig fs))
    66    | Some x \<Rightarrow> frs = []" 
    66    | Some x \<Rightarrow> frs = []" 
    67 
    67 
    68 
    68 
    69 syntax (xsymbols)
    69 notation (xsymbols)
    70  correct_state :: "[jvm_prog,prog_type,jvm_state] \<Rightarrow> bool"
    70  correct_state  ("_,_ \<turnstile>JVM _ \<surd>"  [51,51] 50)
    71                   ("_,_ \<turnstile>JVM _ \<surd>"  [51,51] 50)
       
    72 
    71 
    73 
    72 
    74 lemma sup_ty_opt_OK:
    73 lemma sup_ty_opt_OK:
    75   "(G \<turnstile> X <=o (OK T')) = (\<exists>T. X = OK T \<and> G \<turnstile> T \<preceq> T')"
    74   "(G \<turnstile> X <=o (OK T')) = (\<exists>T. X = OK T \<and> G \<turnstile> T \<preceq> T')"
    76   apply (cases X)
    75   apply (cases X)