src/HOL/Statespace/StateFun.thy
changeset 63167 0909deb8059b
parent 62390 842917225d56
--- a/src/HOL/Statespace/StateFun.thy	Thu May 26 16:57:14 2016 +0200
+++ b/src/HOL/Statespace/StateFun.thy	Thu May 26 17:51:22 2016 +0200
@@ -2,13 +2,13 @@
     Author:     Norbert Schirmer, TU Muenchen
 *)
 
-section {* State Space Representation as Function \label{sec:StateFun}*}
+section \<open>State Space Representation as Function \label{sec:StateFun}\<close>
 
 theory StateFun imports DistinctTreeProver 
 begin
 
 
-text {* The state space is represented as a function from names to
+text \<open>The state space is represented as a function from names to
 values. We neither fix the type of names nor the type of values. We
 define lookup and update functions and provide simprocs that simplify
 expressions containing these, similar to HOL-records.
@@ -20,7 +20,7 @@
 
 The update is actually generalized to a map function. The map supplies
 better compositionality, especially if you think of nested state
-spaces.  *} 
+spaces.\<close> 
 
 definition K_statefun :: "'a \<Rightarrow> 'b \<Rightarrow> 'a" where "K_statefun c x \<equiv> c"