reflexive nbe equation for equality on String.literal
authorhaftmann
Tue, 11 Jun 2013 21:07:53 +0200
changeset 52365 95186e6e4bf4
parent 52364 3bed446c305b
child 52366 ff89424b5094
reflexive nbe equation for equality on String.literal
src/HOL/String.thy
--- a/src/HOL/String.thy	Mon Jun 10 20:43:17 2013 +0200
+++ b/src/HOL/String.thy	Tue Jun 11 21:07:53 2013 +0200
@@ -382,6 +382,11 @@
 
 end
 
+lemma [code nbe]:
+  fixes s :: "String.literal"
+  shows "HOL.equal s s \<longleftrightarrow> True"
+  by (simp add: equal)
+
 lemma STR_inject' [simp]:
   "STR xs = STR ys \<longleftrightarrow> xs = ys"
   by (simp add: STR_inject)