src/HOL/IMP/Procs_Dyn_Vars_Dyn.thy
changeset 45212 e87feee00a4c
parent 44923 b80108b346a9
child 47818 151d137f1095
equal deleted inserted replaced
45211:3dd426ae6bea 45212:e87feee00a4c
     1 theory Procs_Dyn_Vars_Dyn imports Procs
     1 theory Procs_Dyn_Vars_Dyn imports Procs
     2 begin
     2 begin
     3 
     3 
     4 subsubsection "Dynamic Scoping of Procedures and Variables"
     4 subsubsection "Dynamic Scoping of Procedures and Variables"
     5 
     5 
     6 type_synonym penv = "name \<Rightarrow> com"
     6 type_synonym penv = "pname \<Rightarrow> com"
     7 
     7 
     8 inductive
     8 inductive
     9   big_step :: "penv \<Rightarrow> com \<times> state \<Rightarrow> state \<Rightarrow> bool" ("_ \<turnstile> _ \<Rightarrow> _" [60,0,60] 55)
     9   big_step :: "penv \<Rightarrow> com \<times> state \<Rightarrow> state \<Rightarrow> bool" ("_ \<turnstile> _ \<Rightarrow> _" [60,0,60] 55)
    10 where
    10 where
    11 Skip:    "pe \<turnstile> (SKIP,s) \<Rightarrow> s" |
    11 Skip:    "pe \<turnstile> (SKIP,s) \<Rightarrow> s" |