src/HOL/Code_Evaluation.thy
changeset 60758 d8d85a8172b5
parent 59484 a130ae7a9398
child 61076 bdc1e2f0a86a
--- a/src/HOL/Code_Evaluation.thy	Sat Jul 18 21:44:18 2015 +0200
+++ b/src/HOL/Code_Evaluation.thy	Sat Jul 18 22:58:50 2015 +0200
@@ -2,16 +2,16 @@
     Author:     Florian Haftmann, TU Muenchen
 *)
 
-section {* Term evaluation using the generic code generator *}
+section \<open>Term evaluation using the generic code generator\<close>
 
 theory Code_Evaluation
 imports Typerep Limited_Sequence
 keywords "value" :: diag
 begin
 
-subsection {* Term representation *}
+subsection \<open>Term representation\<close>
 
-subsubsection {* Terms and class @{text term_of} *}
+subsubsection \<open>Terms and class @{text term_of}\<close>
 
 datatype (plugins only: code extraction) "term" = dummy_term
 
@@ -44,7 +44,7 @@
   by (simp only: valapp_def fst_conv snd_conv)
 
 
-subsubsection {* Syntax *}
+subsubsection \<open>Syntax\<close>
 
 definition termify :: "'a \<Rightarrow> term" where
   [code del]: "termify x = dummy_term"
@@ -66,7 +66,7 @@
   and valapp (infixl "{\<cdot>}" 70)
 
 
-subsection {* Tools setup and evaluation *}
+subsection \<open>Tools setup and evaluation\<close>
 
 lemma eq_eq_TrueD:
   assumes "(x \<equiv> y) \<equiv> Trueprop True"
@@ -87,7 +87,7 @@
 ML_file "~~/src/HOL/Tools/value.ML"
 
 
-subsection {* @{text term_of} instances *}
+subsection \<open>@{text term_of} instances\<close>
 
 instantiation "fun" :: (typerep, typerep) term_of
 begin
@@ -138,12 +138,12 @@
 code_reserved Eval HOLogic
 
 
-subsection {* Generic reification *}
+subsection \<open>Generic reification\<close>
 
 ML_file "~~/src/HOL/Tools/reification.ML"
 
 
-subsection {* Diagnostic *}
+subsection \<open>Diagnostic\<close>
 
 definition tracing :: "String.literal \<Rightarrow> 'a \<Rightarrow> 'a" where
   [code del]: "tracing s x = x"