src/HOL/ex/String.ML
author lcp
Thu, 29 Jun 1995 16:16:24 +0200
changeset 1167 cbd32a0f2f41
parent 969 b051e2fc2e34
child 1266 3ae9fe3c0f68
permissions -rw-r--r--
New theory and proofs including preorder, inorder, ..., initially from ZF/ex/BT. Demonstrates datatypes and primrec.

val string_ss = list_ss addsimps (String.nibble.simps @ String.char.simps);

goal String.thy "hd(''ABCD'') = CHR ''A''";
by(simp_tac string_ss 1);
result();

goal String.thy "hd(''ABCD'') ~= CHR ''B''";
by(simp_tac string_ss 1);
result();

goal String.thy "''ABCD'' ~= ''ABCX''";
by(simp_tac string_ss 1);
result();

goal String.thy "''ABCD'' = ''ABCD''";
by(simp_tac string_ss 1);
result();

goal String.thy
  "''ABCDEFGHIJKLMNOPQRSTUVWXYZ'' ~= ''ABCDEFGHIJKLMNOPQRSTUVWXY''";
by(simp_tac string_ss 1);
result();