src/HOL/ex/StringEx.thy
author wenzelm
Thu, 16 Feb 2006 18:25:54 +0100
changeset 19070 99001616e0e2
parent 17388 495c799df31d
permissions -rw-r--r--
derived specifications: definition, abbreviation, axiomatization;

(* $Id$ *)

header {* String examples *}

theory StringEx imports Main begin

lemma "hd ''ABCD'' = CHR ''A''"
  by simp

lemma "hd ''ABCD'' \<noteq> CHR ''B''"
  by simp

lemma "''ABCD'' \<noteq> ''ABCX''"
  by simp

lemma "''ABCD'' = ''ABCD''"
  by simp

lemma "''ABCDEFGHIJKLMNOPQRSTUVWXYZ'' \<noteq>
  ''ABCDEFGHIJKLMNOPQRSTUVWXY''"
  by simp

lemma "set ''Foobar'' = {CHR ''F'', CHR ''a'', CHR ''b'', CHR ''o'', CHR ''r''}"
  by (simp add: insert_commute)

lemma "set ''Foobar'' = ?X"
  by (simp add: insert_commute)

end