fixed postprocessing for term presentation in quickcheck; tuned spacing
authorbulwahn
Fri, 25 Mar 2011 11:19:00 +0100
changeset 42110 17e0cd9bc259
parent 42109 f5950b976076
child 42111 d1c761375a75
fixed postprocessing for term presentation in quickcheck; tuned spacing
src/HOL/Tools/Quickcheck/quickcheck_common.ML
--- a/src/HOL/Tools/Quickcheck/quickcheck_common.ML	Thu Mar 24 22:12:38 2011 +0100
+++ b/src/HOL/Tools/Quickcheck/quickcheck_common.ML	Fri Mar 25 11:19:00 2011 +0100
@@ -98,7 +98,7 @@
     fun map_Abs f t =
       case t of Abs (x, T, t') => Abs (x, T, f t') | _ => raise TERM ("map_Abs", [t]) 
     fun process_args t = case strip_comb t of
-      (c as Const (_, _), ts) => list_comb (c, map post_process_term ts) 
+      (c as Const (_, _), ts) => list_comb (c, map post_process_term ts)
   in
     case fastype_of t of
       Type (@{type_name fun}, [T1, T2]) =>
@@ -108,15 +108,15 @@
             |> (case T2 of
               @{typ bool} => 
                 (case t of
-                   Abs(_, _, @{const True}) => fst #> rev #> make_set T1
-                 | Abs(_, _, @{const False}) => fst #> rev #> make_coset T1
+                   Abs(_, _, @{const False}) => fst #> rev #> make_set T1
+                 | Abs(_, _, @{const True}) => fst #> rev #> make_coset T1
                  | Abs(_, _, Const (@{const_name undefined}, _)) => fst #> rev #> make_set T1
                  | _ => raise TERM ("post_process_term", [t]))
             | Type (@{type_name option}, _) =>
                 (case t of
-                  Abs(_, _, Const(@{const_name None}, _)) => fst #> make_map T1 T2
+                  Abs(_, _, Const (@{const_name None}, _)) => fst #> make_map T1 T2
                 | Abs(_, _, Const (@{const_name undefined}, _)) => fst #> make_map T1 T2
-                | _ => make_fun_upds T1 T2) 
+                | _ => make_fun_upds T1 T2)
             | _ => make_fun_upds T1 T2)
         | NONE => process_args t)
     | _ => process_args t