ex/pl.ML
changeset 48 21291189b51e
parent 0 7949f97df77a
child 56 385d51d74f71
--- a/ex/pl.ML	Thu Feb 24 14:45:57 1994 +0100
+++ b/ex/pl.ML	Wed Mar 02 12:26:55 1994 +0100
@@ -158,7 +158,7 @@
 by (simp_tac pl_ss 1);
 val hyps_false = result();
 
-goalw PL.thy [hyps_def] "hyps(#v,tt) = {if(v:tt, #v, #v->false)}";
+goalw PL.thy [hyps_def] "hyps(#v,tt) = {if(v:tt, #v, (#v)->false)}";
 by (simp_tac pl_ss 1);
 val hyps_var = result();
 
@@ -250,7 +250,7 @@
 
 (*For the case hyps(p,t)-insert(#v,Y) |- p;
   we also have hyps(p,t)-{#v} <= hyps(p, t-{v}) *)
-goal PL.thy "!p.hyps(p, t-{v}) <= insert(#v->false, hyps(p,t)-{#v})";
+goal PL.thy "!p.hyps(p, t-{v}) <= insert((#v)->false, hyps(p,t)-{#v})";
 by (rtac pl_ind 1);
 by (simp_tac pl_ss 1);
 by (simp_tac (pl_ss setloop (split_tac [expand_if])) 1);
@@ -260,8 +260,8 @@
 val hyps_Diff = result() RS spec;
 
 (*For the case hyps(p,t)-insert(#v -> false,Y) |- p;
-  we also have hyps(p,t)-{#v->false} <= hyps(p, insert(v,t)) *)
-goal PL.thy "!p.hyps(p, insert(v,t)) <= insert(#v, hyps(p,t)-{#v->false})";
+  we also have hyps(p,t)-{(#v)->false} <= hyps(p, insert(v,t)) *)
+goal PL.thy "!p.hyps(p, insert(v,t)) <= insert(#v, hyps(p,t)-{(#v)->false})";
 by (rtac pl_ind 1);
 by (simp_tac pl_ss 1);
 by (simp_tac (pl_ss setloop (split_tac [expand_if])) 1);
@@ -282,7 +282,7 @@
 
 (*The set hyps(p,t) is finite, and elements have the form #v or #v->false;
  could probably prove the stronger hyps(p,t) : Fin(hyps(p,{}) Un hyps(p,nat))*)
-goal PL.thy "!p.hyps(p,t) : Fin(UN v:{x.True}. {#v, #v->false})";
+goal PL.thy "!p.hyps(p,t) : Fin(UN v:{x.True}. {#v, (#v)->false})";
 by (rtac pl_ind 1);
 by (ALLGOALS (simp_tac (pl_ss setloop (split_tac [expand_if])) THEN'
               fast_tac (set_cs addSIs [Fin_0I, Fin_insertI, Fin_UnI])));