constant "chars" of all characters
authorhaftmann
Mon, 08 Jun 2009 09:22:47 +0200
changeset 31486 bee3b47e1516
parent 31485 259a3c90016e
child 31504 0566495a3986
constant "chars" of all characters
src/HOL/Library/Fin_Fun.thy
--- a/src/HOL/Library/Fin_Fun.thy	Mon Jun 08 08:38:53 2009 +0200
+++ b/src/HOL/Library/Fin_Fun.thy	Mon Jun 08 09:22:47 2009 +0200
@@ -1186,10 +1186,10 @@
 proof -
   from enum_distinct
   have "card (set (enum :: char list)) = length (enum :: char list)"
-    by -(rule distinct_card)
+    by - (rule distinct_card)
   also have "set enum = (UNIV :: char set)" by auto
-  also note enum_char
-  finally show ?thesis by simp
+  also note enum_chars
+  finally show ?thesis by (simp add: chars_def)
 qed
 
 instantiation char :: card_UNIV begin