add translation for wildcard pattern
authorhuffman
Thu, 03 Nov 2005 01:28:22 +0100
changeset 18079 9d4d70b175fd
parent 18078 20e5a6440790
child 18080 c1a7490ee3ff
add translation for wildcard pattern
src/HOLCF/Cfun.thy
--- a/src/HOLCF/Cfun.thy	Thu Nov 03 01:11:39 2005 +0100
+++ b/src/HOLCF/Cfun.thy	Thu Nov 03 01:28:22 2005 +0100
@@ -86,6 +86,9 @@
   in [("_cabs", cabs_ast_tr')] end;
 *}
 
+translations
+  "\<Lambda> _. t" == "Abs_CFun (\<lambda> _. t)"
+
 subsection {* Continuous function space is pointed *}
 
 lemma UU_CFun: "\<bottom> \<in> CFun"