src/HOL/Statespace/StateSpaceLocale.thy
author blanchet
Wed, 02 Jun 2010 15:18:48 +0200
changeset 37321 9d7cfae95b30
parent 29247 95d3a82857e5
child 38838 62f6ba39b3d4
permissions -rw-r--r--
honor "xsymbols"

(*  Title:      StateSpaceLocale.thy
    ID:         $Id$
    Author:     Norbert Schirmer, TU Muenchen
*)

header {* Setup for State Space Locales \label{sec:StateSpaceLocale}*}

theory StateSpaceLocale imports StateFun 
uses "state_space.ML" "state_fun.ML"
begin

setup StateFun.setup

text {* For every type that is to be stored in a state space, an
instance of this locale is imported in order convert the abstract and
concrete values.*}


locale project_inject =
 fixes project :: "'value \<Rightarrow> 'a"
 and   "inject":: "'a \<Rightarrow> 'value"
 assumes project_inject_cancel [statefun_simp]: "project (inject x) = x"

lemma (in project_inject)
 ex_project [statefun_simp]: "\<exists>v. project v = x"
  apply (rule_tac x= "inject x" in exI)
  apply (simp add: project_inject_cancel)
  done

lemma (in project_inject)
 project_inject_comp_id [statefun_simp]: "project \<circ> inject = id"
  by (rule ext) (simp add: project_inject_cancel)

lemma (in project_inject)
 project_inject_comp_cancel[statefun_simp]: "f \<circ> project \<circ> inject = f"
  by (rule ext) (simp add: project_inject_cancel)



end