src/HOL/Proofs/Lambda/ListBeta.thy
changeset 61986 2461779da2b8
parent 58889 5b7a9633cfa8
child 61987 305baa3fc220
--- a/src/HOL/Proofs/Lambda/ListBeta.thy	Wed Dec 30 18:24:36 2015 +0100
+++ b/src/HOL/Proofs/Lambda/ListBeta.thy	Wed Dec 30 18:25:39 2015 +0100
@@ -3,13 +3,13 @@
     Copyright   1998 TU Muenchen
 *)
 
-section {* Lifting beta-reduction to lists *}
+section \<open>Lifting beta-reduction to lists\<close>
 
 theory ListBeta imports ListApplication ListOrder begin
 
-text {*
+text \<open>
   Lifting beta-reduction to lists of terms, reducing exactly one element.
-*}
+\<close>
 
 abbreviation
   list_beta :: "dB list => dB list => bool"  (infixl "=>" 50) where