src/HOL/Isar_Examples/Group_Context.thy
changeset 58614 7338eb25226c
parent 55656 eb07b0acbebc
child 58882 6e2010ab8bd9
--- a/src/HOL/Isar_Examples/Group_Context.thy	Tue Oct 07 20:43:18 2014 +0200
+++ b/src/HOL/Isar_Examples/Group_Context.thy	Tue Oct 07 20:59:46 2014 +0200
@@ -2,13 +2,13 @@
     Author:     Makarius
 *)
 
-header {* Some algebraic identities derived from group axioms -- theory context version *}
+header \<open>Some algebraic identities derived from group axioms -- theory context version\<close>
 
 theory Group_Context
 imports Main
 begin
 
-text {* hypothetical group axiomatization *}
+text \<open>hypothetical group axiomatization\<close>
 
 context
   fixes prod :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "**" 70)
@@ -19,7 +19,7 @@
     and left_inverse: "inverse x ** x = one"
 begin
 
-text {* some consequences *}
+text \<open>some consequences\<close>
 
 lemma right_inverse: "x ** inverse x = one"
 proof -