src/HOL/Bali/Trans.thy
changeset 16417 9bc16273c2d4
parent 14981 e73f8140af78
child 21765 89275a3ed7be
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     6 execution of Java expressions and statements
     6 execution of Java expressions and statements
     7 
     7 
     8 PRELIMINARY!!!!!!!!
     8 PRELIMINARY!!!!!!!!
     9 *)
     9 *)
    10 
    10 
    11 theory Trans = Evaln:
    11 theory Trans imports Evaln begin
    12 
    12 
    13 constdefs groundVar:: "var \<Rightarrow> bool"
    13 constdefs groundVar:: "var \<Rightarrow> bool"
    14 "groundVar v \<equiv> (case v of
    14 "groundVar v \<equiv> (case v of
    15                    LVar ln \<Rightarrow> True
    15                    LVar ln \<Rightarrow> True
    16                  | {accC,statDeclC,stat}e..fn \<Rightarrow> \<exists> a. e=Lit a
    16                  | {accC,statDeclC,stat}e..fn \<Rightarrow> \<exists> a. e=Lit a