src/HOL/Quickcheck_Exhaustive.thy
changeset 45684 3d6ee9c7d7ef
parent 45450 dc2236b19a3d
child 45697 3b7c35a08723
--- a/src/HOL/Quickcheck_Exhaustive.thy	Wed Nov 30 09:21:07 2011 +0100
+++ b/src/HOL/Quickcheck_Exhaustive.thy	Wed Nov 30 09:21:09 2011 +0100
@@ -530,6 +530,15 @@
 code_const catch_match 
   (Quickcheck "(_) handle Match => _")
 
+definition catch_match' :: "term => term => term"
+where
+  [code del]: "catch_match' t1 t2 = (SOME t. t = t1 \<or> t = t2)"
+
+code_const catch_match'
+  (Quickcheck "(_) handle Match => _")
+
+consts unknown :: "'a" ("?")
+ 
 use "Tools/Quickcheck/exhaustive_generators.ML"
 
 setup {* Exhaustive_Generators.setup *}