src/HOLCF/Fun2.ML
changeset 3842 b55686a7b22c
parent 3323 194ae2e0c193
child 4098 71e05eb27fb6
--- a/src/HOLCF/Fun2.ML	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOLCF/Fun2.ML	Fri Oct 10 19:02:28 1997 +0200
@@ -9,7 +9,7 @@
 open Fun2;
 
 (* for compatibility with old HOLCF-Version *)
-qed_goal "inst_fun_po" thy "(op <<)=(%f g.!x.f x << g x)"
+qed_goal "inst_fun_po" thy "(op <<)=(%f g.!x. f x << g x)"
  (fn prems => 
         [
 	(fold_goals_tac [less_fun_def]),
@@ -20,7 +20,7 @@
 (* Type 'a::term => 'b::pcpo is pointed                                     *)
 (* ------------------------------------------------------------------------ *)
 
-qed_goal "minimal_fun" thy "(%z.UU) << x"
+qed_goal "minimal_fun" thy "(%z. UU) << x"
 (fn prems =>
         [
         (simp_tac (!simpset addsimps [inst_fun_po,minimal]) 1)
@@ -28,10 +28,10 @@
 
 bind_thm ("UU_fun_def",minimal_fun RS minimal2UU RS sym);
 
-qed_goal "least_fun" thy "? x::'a=>'b::pcpo.!y.x<<y"
+qed_goal "least_fun" thy "? x::'a=>'b::pcpo.!y. x<<y"
 (fn prems =>
         [
-        (res_inst_tac [("x","(%z.UU)")] exI 1),
+        (res_inst_tac [("x","(%z. UU)")] exI 1),
         (rtac (minimal_fun RS allI) 1)
         ]);
 
@@ -52,7 +52,7 @@
 (* ------------------------------------------------------------------------ *)
 
 qed_goal "ch2ch_fun" thy 
-        "is_chain(S::nat=>('a=>'b::po)) ==> is_chain(% i.S(i)(x))"
+        "is_chain(S::nat=>('a=>'b::po)) ==> is_chain(% i. S(i)(x))"
 (fn prems =>
         [
         (cut_facts_tac prems 1),
@@ -87,7 +87,7 @@
 
 qed_goal "lub_fun"  Fun2.thy
         "is_chain(S::nat=>('a::term => 'b::cpo)) ==> \
-\        range(S) <<| (% x.lub(range(% i.S(i)(x))))"
+\        range(S) <<| (% x. lub(range(% i. S(i)(x))))"
 (fn prems =>
         [
         (cut_facts_tac prems 1),