src/HOL/NanoJava/Equivalence.thy
changeset 16417 9bc16273c2d4
parent 14565 c6dc17aab88a
child 23755 1c4672d130b1
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4     Copyright   2001 Technische Universitaet Muenchen
     4     Copyright   2001 Technische Universitaet Muenchen
     5 *)
     5 *)
     6 
     6 
     7 header "Equivalence of Operational and Axiomatic Semantics"
     7 header "Equivalence of Operational and Axiomatic Semantics"
     8 
     8 
     9 theory Equivalence = OpSem + AxSem:
     9 theory Equivalence imports OpSem AxSem begin
    10 
    10 
    11 subsection "Validity"
    11 subsection "Validity"
    12 
    12 
    13 constdefs
    13 constdefs
    14   valid   :: "[assn,stmt, assn] => bool"  ("|= {(1_)}/ (_)/ {(1_)}" [3,90,3] 60)
    14   valid   :: "[assn,stmt, assn] => bool"  ("|= {(1_)}/ (_)/ {(1_)}" [3,90,3] 60)