src/CTT/Bool.thy
changeset 60770 240563fbf41d
parent 58977 9576b510f6a2
child 61391 2332d9be352b
--- a/src/CTT/Bool.thy	Thu Jul 23 14:20:51 2015 +0200
+++ b/src/CTT/Bool.thy	Thu Jul 23 14:25:05 2015 +0200
@@ -3,7 +3,7 @@
     Copyright   1991  University of Cambridge
 *)
 
-section {* The two-element type (booleans and conditionals) *}
+section \<open>The two-element type (booleans and conditionals)\<close>
 
 theory Bool
 imports CTT
@@ -28,7 +28,7 @@
 lemmas bool_defs = Bool_def true_def false_def cond_def
 
 
-subsection {* Derivation of rules for the type Bool *}
+subsection \<open>Derivation of rules for the type Bool\<close>
 
 (*formation rule*)
 lemma boolF: "Bool type"