src/HOL/String.thy
changeset 44278 1220ecb81e8f
parent 42440 5e7a7343ab11
child 45182 10202ca034b0
--- a/src/HOL/String.thy	Thu Aug 18 13:25:17 2011 +0200
+++ b/src/HOL/String.thy	Thu Aug 18 13:55:26 2011 +0200
@@ -155,7 +155,7 @@
 
 subsection {* Strings as dedicated type *}
 
-typedef (open) literal = "UNIV :: string \<Rightarrow> bool"
+typedef (open) literal = "UNIV :: string set"
   morphisms explode STR ..
 
 instantiation literal :: size