src/HOL/Statespace/StateSpaceLocale.thy
changeset 69913 ca515cf61651
parent 69605 a96320074298
equal deleted inserted replaced
69912:dd55d2c926d9 69913:ca515cf61651
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Setup for State Space Locales \label{sec:StateSpaceLocale}\<close>
     5 section \<open>Setup for State Space Locales \label{sec:StateSpaceLocale}\<close>
     6 
     6 
     7 theory StateSpaceLocale imports StateFun 
     7 theory StateSpaceLocale imports StateFun 
     8 keywords "statespace" :: thy_decl
     8 keywords "statespace" :: thy_defn
     9 begin
     9 begin
    10 
    10 
    11 ML_file \<open>state_space.ML\<close>
    11 ML_file \<open>state_space.ML\<close>
    12 ML_file \<open>state_fun.ML\<close>
    12 ML_file \<open>state_fun.ML\<close>
    13 
    13