diff -r 4a16f8e41879 -r 7338eb25226c src/HOL/Isar_Examples/Group_Context.thy --- 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 \Some algebraic identities derived from group axioms -- theory context version\ theory Group_Context imports Main begin -text {* hypothetical group axiomatization *} +text \hypothetical group axiomatization\ context fixes prod :: "'a \ 'a \ 'a" (infixl "**" 70) @@ -19,7 +19,7 @@ and left_inverse: "inverse x ** x = one" begin -text {* some consequences *} +text \some consequences\ lemma right_inverse: "x ** inverse x = one" proof -