src/HOL/IMP/Big_Step.thy
changeset 59451 86be42bb5174
parent 54192 a5eec4263b3a
child 61337 4645502c3c64
equal deleted inserted replaced
59450:e82c72f3b227 59451:86be42bb5174
     4 
     4 
     5 subsection "Big-Step Semantics of Commands"
     5 subsection "Big-Step Semantics of Commands"
     6 
     6 
     7 text {*
     7 text {*
     8 The big-step semantics is a straight-forward inductive definition
     8 The big-step semantics is a straight-forward inductive definition
     9 with concrete syntax. Note that the first paramenter is a tuple,
     9 with concrete syntax. Note that the first parameter is a tuple,
    10 so the syntax becomes @{text "(c,s) \<Rightarrow> s'"}.
    10 so the syntax becomes @{text "(c,s) \<Rightarrow> s'"}.
    11 *}
    11 *}
    12 
    12 
    13 text_raw{*\snip{BigStepdef}{0}{1}{% *}
    13 text_raw{*\snip{BigStepdef}{0}{1}{% *}
    14 inductive
    14 inductive