src/HOL/Quickcheck_Narrowing.thy
changeset 46589 689311986778
parent 46308 e5abbec2697a
child 46758 4106258260b3
--- a/src/HOL/Quickcheck_Narrowing.thy	Wed Feb 22 12:30:01 2012 +0100
+++ b/src/HOL/Quickcheck_Narrowing.thy	Wed Feb 22 17:22:53 2012 +0100
@@ -8,6 +8,7 @@
   ("Tools/Quickcheck/PNF_Narrowing_Engine.hs")
   ("Tools/Quickcheck/Narrowing_Engine.hs")
   ("Tools/Quickcheck/narrowing_generators.ML")
+  ("Tools/Quickcheck/find_unused_assms.ML")
 begin
 
 subsection {* Counterexample generator *}
@@ -452,10 +453,15 @@
 
 *)
 
+subsection {* The @{text find_unused_assms} command *}
+
+use "Tools/Quickcheck/find_unused_assms.ML"
+
+subsection {* Closing up *}
+
 hide_type code_int narrowing_type narrowing_term cons property
 hide_const int_of of_int nat_of map_cons nth error toEnum marker empty C conv nonEmpty ensure_testable all exists drawn_from around_zero
 hide_const (open) Var Ctr "apply" sum cons
 hide_fact empty_def cons_def conv.simps nonEmpty.simps apply_def sum_def ensure_testable_def all_def exists_def
 
-
 end