src/HOL/Library/IArray.thy
changeset 60500 903bb1495239
parent 59457 c4f044389c28
child 61115 3a4400985780
--- a/src/HOL/Library/IArray.thy	Wed Jun 17 10:57:11 2015 +0200
+++ b/src/HOL/Library/IArray.thy	Wed Jun 17 11:03:05 2015 +0200
@@ -4,14 +4,14 @@
 imports Main
 begin
 
-text{* Immutable arrays are lists wrapped up in an additional constructor.
+text\<open>Immutable arrays are lists wrapped up in an additional constructor.
 There are no update operations. Hence code generation can safely implement
 this type by efficient target language arrays.  Currently only SML is
 provided. Should be extended to other target languages and more operations.
 
 Note that arrays cannot be printed directly but only by turning them into
 lists first. Arrays could be converted back into lists for printing if they
-were wrapped up in an additional constructor. *}
+were wrapped up in an additional constructor.\<close>
 
 datatype 'a iarray = IArray "'a list"