correcting names in Narrowing_Engine and example theory for Quickcheck_Narrowing
authorbulwahn
Mon, 14 Mar 2011 12:34:09 +0100
changeset 41962 27a61a3266d8
parent 41961 fdd37cfcd4a3
child 41963 d8c3b26b3da4
correcting names in Narrowing_Engine and example theory for Quickcheck_Narrowing
src/HOL/Library/Quickcheck_Narrowing.thy
src/HOL/Tools/Quickcheck/Narrowing_Engine.hs
src/HOL/ex/Quickcheck_Narrowing_Examples.thy
--- a/src/HOL/Library/Quickcheck_Narrowing.thy	Mon Mar 14 12:34:08 2011 +0100
+++ b/src/HOL/Library/Quickcheck_Narrowing.thy	Mon Mar 14 12:34:09 2011 +0100
@@ -4,7 +4,8 @@
 
 theory Quickcheck_Narrowing
 imports Main "~~/src/HOL/Library/Code_Char"
-uses ("~~/src/HOL/Tools/Quickcheck/narrowing_generators.ML")
+uses
+  ("~~/src/HOL/Tools/Quickcheck/narrowing_generators.ML")
 begin
 
 subsection {* Counterexample generator *}
--- a/src/HOL/Tools/Quickcheck/Narrowing_Engine.hs	Mon Mar 14 12:34:08 2011 +0100
+++ b/src/HOL/Tools/Quickcheck/Narrowing_Engine.hs	Mon Mar 14 12:34:09 2011 +0100
@@ -89,9 +89,9 @@
   property app = P $ \n d -> Result [] [] (app . reverse);
 };
 
-instance (Term_of a, Serial a, Testable b) => Testable (a -> b) where {
+instance (Term_of a, Narrowing a, Testable b) => Testable (a -> b) where {
   property f = P $ \n d ->
-    let C t c = series d
+    let C t c = narrowing d
         c' = conv c
         r = run (\(x:xs) -> f xs (c' x)) (n+1) d
     in  r { args = Var [n] t : args r, showArgs = (show . term_of . c') : showArgs r };
--- a/src/HOL/ex/Quickcheck_Narrowing_Examples.thy	Mon Mar 14 12:34:08 2011 +0100
+++ b/src/HOL/ex/Quickcheck_Narrowing_Examples.thy	Mon Mar 14 12:34:09 2011 +0100
@@ -115,12 +115,12 @@
                  
 subsection {* Necessary instantiation for quickcheck generator *}
 
-instantiation tree :: (serial) serial
+instantiation tree :: (narrowing) narrowing
 begin
 
-function series_tree
+function narrowing_tree
 where
-  "series_tree d = sum (cons ET) (apply (apply (apply (apply (cons MKT) series) series_tree) series_tree) series) d"
+  "narrowing_tree d = sum (cons ET) (apply (apply (apply (apply (cons MKT) narrowing) narrowing_tree) narrowing_tree) narrowing) d"
 by pat_completeness auto
 
 termination proof (relation "measure nat_of")