equal
deleted
inserted
replaced
117 |
117 |
118 |
118 |
119 text{* |
119 text{* |
120 illustrates Union as well as image |
120 illustrates Union as well as image |
121 *} |
121 *} |
122 lemma "f``A \<union> g``A = (\<Union>x\<in>A. {f x, g x})" |
122 lemma "f`A \<union> g`A = (\<Union>x\<in>A. {f x, g x})" |
123 apply (blast) |
123 apply (blast) |
124 done |
124 done |
125 |
125 |
126 lemma "f `` {(x,y). P x y} = {f(x,y) | x y. P x y}" |
126 lemma "f ` {(x,y). P x y} = {f(x,y) | x y. P x y}" |
127 apply (blast) |
127 apply (blast) |
128 done |
128 done |
129 |
129 |
130 text{*actually a macro!*} |
130 text{*actually a macro!*} |
131 |
131 |
132 lemma "range f = f``UNIV" |
132 lemma "range f = f`UNIV" |
133 apply (blast) |
133 apply (blast) |
134 done |
134 done |
135 |
135 |
136 |
136 |
137 text{* |
137 text{* |