src/HOL/Quickcheck.thy
changeset 48273 65233084e9d7
parent 46976 80123a220219
child 48891 c0eafbd55de3
--- a/src/HOL/Quickcheck.thy	Mon Jul 16 21:20:56 2012 +0200
+++ b/src/HOL/Quickcheck.thy	Tue Jul 17 10:39:39 2012 +0200
@@ -19,7 +19,7 @@
 axiomatization catch_match :: "'a => 'a => 'a"
 
 code_const catch_match 
-  (Quickcheck "(_) handle Match => _")
+  (Quickcheck "((_) handle Match => _)")
 
 subsection {* The @{text random} class *}