tuned;
authorwenzelm
Sat, 14 Jan 2012 18:18:06 +0100
changeset 46216 7fcdb5562461
parent 46215 0da9433f959e
child 46217 7b19666f0e3d
tuned;
src/HOL/Tools/hologic.ML
--- a/src/HOL/Tools/hologic.ML	Sat Jan 14 17:45:04 2012 +0100
+++ b/src/HOL/Tools/hologic.ML	Sat Jan 14 18:18:06 2012 +0100
@@ -255,11 +255,11 @@
 fun dest_eq (Const ("HOL.eq", _) $ lhs $ rhs) = (lhs, rhs)
   | dest_eq t = raise TERM ("dest_eq", [t])
 
-fun all_const T = Const ("HOL.All", [T --> boolT] ---> boolT);
+fun all_const T = Const ("HOL.All", (T --> boolT) --> boolT);
 fun mk_all (x, T, P) = all_const T $ absfree (x, T) P;
 fun list_all (xs, t) = fold_rev (fn (x, T) => fn P => all_const T $ Abs (x, T, P)) xs t;
 
-fun exists_const T = Const ("HOL.Ex", [T --> boolT] ---> boolT);
+fun exists_const T = Const ("HOL.Ex", (T --> boolT) --> boolT);
 fun mk_exists (x, T, P) = exists_const T $ absfree (x, T) P;
 
 fun choice_const T = Const("Hilbert_Choice.Eps", (T --> boolT) --> T);
@@ -270,14 +270,12 @@
 (* binary operations and relations *)
 
 fun mk_binop c (t, u) =
-  let val T = fastype_of t in
-    Const (c, [T, T] ---> T) $ t $ u
-  end;
+  let val T = fastype_of t
+  in Const (c, T --> T --> T) $ t $ u end;
 
 fun mk_binrel c (t, u) =
-  let val T = fastype_of t in
-    Const (c, [T, T] ---> boolT) $ t $ u
-  end;
+  let val T = fastype_of t
+  in Const (c, T --> T --> boolT) $ t $ u end;
 
 (*destruct the application of a binary operator. The dummyT case is a crude
   way of handling polymorphic operators.*)
@@ -307,7 +305,7 @@
 fun dest_prodT (Type ("Product_Type.prod", [T1, T2])) = (T1, T2)
   | dest_prodT T = raise TYPE ("dest_prodT", [T], []);
 
-fun pair_const T1 T2 = Const ("Product_Type.Pair", [T1, T2] ---> mk_prodT (T1, T2));
+fun pair_const T1 T2 = Const ("Product_Type.Pair", T1 --> T2 --> mk_prodT (T1, T2));
 
 fun mk_prod (t1, t2) =
   let val T1 = fastype_of t1 and T2 = fastype_of t2 in