# HG changeset patch # User wenzelm # Date 1004107750 -7200 # Node ID 013d52bb000076e2d788169ad119b753857979e5 # Parent adef41692ab0b97a8ef549fee63558fc62942ea6 tuned; diff -r adef41692ab0 -r 013d52bb0000 src/HOL/Lambda/ListApplication.thy --- a/src/HOL/Lambda/ListApplication.thy Fri Oct 26 16:18:14 2001 +0200 +++ b/src/HOL/Lambda/ListApplication.thy Fri Oct 26 16:49:10 2001 +0200 @@ -11,7 +11,7 @@ syntax "_list_application" :: "dB => dB list => dB" (infixl "$$" 150) syntax (symbols) - "_list_application" :: "dB => dB => dB" (infixl "\<^sub>\\<^sub>\" 150) + "_list_application" :: "dB => dB list => dB" (infixl "\<^sub>\\<^sub>\" 150) translations "t $$ ts" == "foldl (op $) t ts" diff -r adef41692ab0 -r 013d52bb0000 src/HOL/Lambda/Type.thy --- a/src/HOL/Lambda/Type.thy Fri Oct 26 16:18:14 2001 +0200 +++ b/src/HOL/Lambda/Type.thy Fri Oct 26 16:49:10 2001 +0200 @@ -182,8 +182,7 @@ apply auto done -lemma lifts_IT: - "ts \ lists IT \ map (\t. lift t 0) ts \ lists IT" +lemma lifts_IT: "ts \ lists IT \ map (\t. lift t 0) ts \ lists IT" by (induct ts) auto lemma lift_type [intro!]: "e \ t : T \ e\i:U\ \ lift t i : T" @@ -362,7 +361,7 @@ with nT have "e\i:T\ \ Var n \<^sub>\ a \<^sub>\\<^sub>\ as : T'" by simp then obtain Ts where headT: "e\i:T\ \ Var n \<^sub>\ a : Ts \ T'" - and argsT: "(e\i:T\) \ as : Ts" + and argsT: "e\i:T\ \ as : Ts" by (rule list_app_typeE) from headT obtain T'' where varT: "e\i:T\ \ Var n : T'' \ Ts \ T'" @@ -418,7 +417,7 @@ by (rule typing.Var) simp moreover from uT argsT have "e \ map (\t. t[u/i]) as : Ts" by (rule substs_lemma) - hence "(e\0:Ts \ T'\) \ ?ls as : Ts" + hence "e\0:Ts \ T'\ \ ?ls as : Ts" by (rule lift_typings) ultimately show "e\0:Ts \ T'\ \ Var 0 \<^sub>\\<^sub>\ ?ls as : T'" by (rule list_app_typeI) @@ -433,7 +432,7 @@ next case False from Var have "rs \ lists {t. ?R t}" by simp - moreover from nT obtain Ts where "(e\i:T\) \ rs : Ts" + moreover from nT obtain Ts where "e\i:T\ \ rs : Ts" by (rule list_app_typeE) hence "rs \ lists ?ty" by (rule lists_typings) ultimately have "rs \ lists ({t. ?R t} \ ?ty)"