src/HOL/String.thy
changeset 45141 1220ecb81e8f
parent 43311 5e7a7343ab11
child 46053 10202ca034b0
     1.1 --- a/src/HOL/String.thy	Thu Aug 18 13:25:17 2011 +0200
     1.2 +++ b/src/HOL/String.thy	Thu Aug 18 13:55:26 2011 +0200
     1.3 @@ -155,7 +155,7 @@
     1.4  
     1.5  subsection {* Strings as dedicated type *}
     1.6  
     1.7 -typedef (open) literal = "UNIV :: string \<Rightarrow> bool"
     1.8 +typedef (open) literal = "UNIV :: string set"
     1.9    morphisms explode STR ..
    1.10  
    1.11  instantiation literal :: size