src/HOL/MicroJava/BV/LBVCorrect.thy
changeset 13365 a2c4faad4d35
parent 13215 072a77989ce0
child 13649 0f562a70c07d
equal deleted inserted replaced
13364:d3c7d05d8839 13365:a2c4faad4d35
     6 
     6 
     7 header {* \isaheader{Correctness of the LBV} *}
     7 header {* \isaheader{Correctness of the LBV} *}
     8 
     8 
     9 theory LBVCorrect = LBVSpec + Typing_Framework:
     9 theory LBVCorrect = LBVSpec + Typing_Framework:
    10 
    10 
    11 locale lbvs = lbv +
    11 locale (open) lbvs = lbv +
    12   fixes s0  :: 'a
    12   fixes s0  :: 'a
    13   fixes c   :: "'a list"
    13   fixes c   :: "'a list"
    14   fixes ins :: "'b list"
    14   fixes ins :: "'b list"
    15   fixes phi :: "'a list" ("\<phi>")
    15   fixes phi :: "'a list" ("\<phi>")
    16   defines phi_def:
    16   defines phi_def: