adding some rules to quickcheck's preprocessing
authorbulwahn
Tue, 24 Jan 2012 09:13:24 +0100
changeset 46327 ecda23528833
parent 46326 9a5d8e7684e5
child 46328 fd21bbcbe61b
child 46329 cf3b387ba667
adding some rules to quickcheck's preprocessing
src/HOL/Tools/Quickcheck/quickcheck_common.ML
--- a/src/HOL/Tools/Quickcheck/quickcheck_common.ML	Tue Jan 24 09:12:29 2012 +0100
+++ b/src/HOL/Tools/Quickcheck/quickcheck_common.ML	Tue Jan 24 09:13:24 2012 +0100
@@ -262,7 +262,8 @@
     val thy = Proof_Context.theory_of ctxt
     val dest = HOLogic.dest_eq o HOLogic.dest_Trueprop o Thm.prop_of
     val rewrs = map (swap o dest) @{thms all_simps} @
-      (map dest [@{thm not_ex}, @{thm not_all}, @{thm imp_conjL}, @{thm fun_eq_iff}])
+      (map dest [@{thm not_ex}, @{thm not_all}, @{thm imp_conjL}, @{thm fun_eq_iff},
+        @{thm bot_fun_def}, @{thm less_bool_def}])
     val t' = Pattern.rewrite_term thy rewrs [] (Object_Logic.atomize_term thy t)
     val (vs, body) = strip_all t'
     val vs' = Variable.variant_frees ctxt [t'] vs