change match_bottom_simps to produce if-then-else, making more uses of bottom-patterns work with fixrec
authorhuffman
Sun, 28 Nov 2010 07:29:32 -0800
changeset 40795 c52cd8bc426d
parent 40794 d28d41ee4cef
child 40796 aeeb3e61e3af
change match_bottom_simps to produce if-then-else, making more uses of bottom-patterns work with fixrec
src/HOL/HOLCF/Fixrec.thy
--- a/src/HOL/HOLCF/Fixrec.thy	Sat Nov 27 22:48:08 2010 -0800
+++ b/src/HOL/HOLCF/Fixrec.thy	Sun Nov 28 07:29:32 2010 -0800
@@ -150,9 +150,8 @@
   "match_FF = (\<Lambda> x k. If x then fail else k)"
 
 lemma match_bottom_simps [simp]:
-  "match_bottom\<cdot>\<bottom>\<cdot>k = \<bottom>"
-  "x \<noteq> \<bottom> \<Longrightarrow> match_bottom\<cdot>x\<cdot>k = fail"
-by (simp_all add: match_bottom_def)
+  "match_bottom\<cdot>x\<cdot>k = (if x = \<bottom> then \<bottom> else fail)"
+by (simp add: match_bottom_def)
 
 lemma match_Pair_simps [simp]:
   "match_Pair\<cdot>(x, y)\<cdot>k = k\<cdot>x\<cdot>y"