src/HOLCF/ex/Pattern_Match.thy
changeset 40322 707eb30e8a53
parent 40026 8f8f18a88685
child 40326 73d45866dbda
--- a/src/HOLCF/ex/Pattern_Match.thy	Wed Oct 27 13:54:18 2010 -0700
+++ b/src/HOLCF/ex/Pattern_Match.thy	Wed Oct 27 14:15:54 2010 -0700
@@ -184,11 +184,11 @@
 
 definition
   TT_pat :: "(tr, unit) pat" where
-  "TT_pat = (\<Lambda> b. If b then succeed\<cdot>() else fail fi)"
+  "TT_pat = (\<Lambda> b. If b then succeed\<cdot>() else fail)"
 
 definition
   FF_pat :: "(tr, unit) pat" where
-  "FF_pat = (\<Lambda> b. If b then fail else succeed\<cdot>() fi)"
+  "FF_pat = (\<Lambda> b. If b then fail else succeed\<cdot>())"
 
 definition
   ONE_pat :: "(one, unit) pat" where