src/HOL/BNF_Greatest_Fixpoint.thy
changeset 60758 d8d85a8172b5
parent 58889 5b7a9633cfa8
child 61032 b57df8eecad6
--- a/src/HOL/BNF_Greatest_Fixpoint.thy	Sat Jul 18 21:44:18 2015 +0200
+++ b/src/HOL/BNF_Greatest_Fixpoint.thy	Sat Jul 18 22:58:50 2015 +0200
@@ -7,7 +7,7 @@
 Greatest fixpoint (codatatype) operation on bounded natural functors.
 *)
 
-section {* Greatest Fixpoint (Codatatype) Operation on Bounded Natural Functors *}
+section \<open>Greatest Fixpoint (Codatatype) Operation on Bounded Natural Functors\<close>
 
 theory BNF_Greatest_Fixpoint
 imports BNF_Fixpoint_Base String
@@ -17,7 +17,7 @@
   "primcorec" :: thy_decl
 begin
 
-setup {* Sign.const_alias @{binding proj} @{const_name Equiv_Relations.proj} *}
+setup \<open>Sign.const_alias @{binding proj} @{const_name Equiv_Relations.proj}\<close>
 
 lemma one_pointE: "\<lbrakk>\<And>x. s = x \<Longrightarrow> P\<rbrakk> \<Longrightarrow> P"
   by simp
@@ -240,7 +240,7 @@
   unfolding rel_fun_def image2p_def by auto
 
 
-subsection {* Equivalence relations, quotients, and Hilbert's choice *}
+subsection \<open>Equivalence relations, quotients, and Hilbert's choice\<close>
 
 lemma equiv_Eps_in:
 "\<lbrakk>equiv A r; X \<in> A//r\<rbrakk> \<Longrightarrow> Eps (%x. x \<in> X) \<in> X"