Theory WWellForm

Up to index of Isabelle/HOL/Jinja

theory WWellForm
imports WellForm Expr
(*  Title:      Jinja/J/WWellForm.thy

Author: Tobias Nipkow
Copyright 2003 Technische Universitaet Muenchen
*)


header {* \isaheader{Weak well-formedness of Jinja programs} *}

theory WWellForm imports "../Common/WellForm" Expr begin

definition wwf_J_mdecl :: "J_prog => cname => J_mb mdecl => bool"
where
"wwf_J_mdecl P C ≡ λ(M,Ts,T,(pns,body)).
length Ts = length pns ∧ distinct pns ∧ this ∉ set pns ∧ fv body ⊆ {this} ∪ set pns"


lemma wwf_J_mdecl[simp]:
"wwf_J_mdecl P C (M,Ts,T,pns,body) =
(length Ts = length pns ∧ distinct pns ∧ this ∉ set pns ∧ fv body ⊆ {this} ∪ set pns)"

(*<*)by(simp add:wwf_J_mdecl_def)(*>*)

abbreviation
wwf_J_prog :: "J_prog => bool" where
"wwf_J_prog == wf_prog wwf_J_mdecl"

end