--- a/src/HOL/Quickcheck_Examples/Quickcheck_Narrowing_Examples.thy Sat Mar 24 16:27:04 2012 +0100
+++ b/src/HOL/Quickcheck_Examples/Quickcheck_Narrowing_Examples.thy Sun Mar 25 20:15:39 2012 +0200
@@ -79,15 +79,14 @@
quickcheck[tester = narrowing, finite_types = false, default_type = nat, expect = counterexample]
oops
-(* FIXME: integer has strange representation! *)
lemma "rev xs = xs"
quickcheck[tester = narrowing, finite_types = false, default_type = int, expect = counterexample]
oops
-(*
+
lemma "rev xs = xs"
quickcheck[tester = narrowing, finite_types = true, expect = counterexample]
oops
-*)
+
subsection {* Simple examples with functions *}
lemma "map f xs = map g xs"