File tree Expand file tree Collapse file tree 2 files changed +9
-9
lines changed Expand file tree Collapse file tree 2 files changed +9
-9
lines changed Original file line number Diff line number Diff line change @@ -358,11 +358,11 @@ Variable f:point_set X -> point_set Y -> point_set Z.
358
358
359
359
Definition continuous_2arg :=
360
360
continuous (fun p:point_set X * point_set Y =>
361
- let (x,y):=p in f x y )
361
+ f (fst p) (snd p) )
362
362
(X:=ProductTopology2 X Y).
363
363
Definition continuous_at_2arg (x:point_set X) (y:point_set Y) :=
364
364
continuous_at (fun p:point_set X * point_set Y =>
365
- let (x,y):=p in f x y ) (x, y)
365
+ f (fst p) (snd p) ) (x, y)
366
366
(X:=ProductTopology2 X Y).
367
367
368
368
Lemma continuous_2arg_func_continuous_everywhere:
@@ -398,9 +398,10 @@ Lemma continuous_composition_at_2arg:
398
398
continuous_at (fun w:point_set W => f (g w) (h w)) w.
399
399
Proof .
400
400
intros.
401
+ red in H.
401
402
apply (continuous_composition_at
402
403
(fun p:point_set (ProductTopology2 X Y) =>
403
- let (x,y):=p in f x y )
404
+ f (fst p) (snd p) )
404
405
(fun w:point_set W => (g w, h w))); trivial.
405
406
now apply product2_map_continuous_at.
406
407
Qed .
Original file line number Diff line number Diff line change @@ -81,6 +81,7 @@ apply continuous_at_neighborhood_basis with
81
81
+ destruct x0 as [x' y'],
82
82
H1 as [[[] []]].
83
83
unfold R_metric.
84
+ simpl.
84
85
replace (x'+y' - (x+y)) with ((x'-x) + (y'-y)) by ring.
85
86
apply Rle_lt_trans with (Rabs (x'-x) + Rabs(y'-y)).
86
87
* apply Rabs_triang.
@@ -167,9 +168,8 @@ pose proof (RTop_metrization 0).
167
168
apply continuous_at_neighborhood_basis with
168
169
(metric_topology_neighborhood_basis R_metric 0).
169
170
- apply open_neighborhood_basis_is_neighborhood_basis.
170
- replace (0*0) with 0 by auto with real.
171
- apply H.
172
-
171
+ simpl. rewrite Rmult_0_r.
172
+ assumption.
173
173
- intros.
174
174
destruct H0.
175
175
exists (characteristic_function_to_ensemble
@@ -192,9 +192,8 @@ apply continuous_at_neighborhood_basis with
192
192
destruct x as [x y].
193
193
destruct H1 as [[] []].
194
194
unfold R_metric in *.
195
- replace (x*y-0) with (x*y) by auto with real.
196
- replace (x-0) with x in H1 by auto with real.
197
- replace (y-0) with y in H2 by auto with real.
195
+ simpl.
196
+ rewrite Rminus_0_r in *.
198
197
rewrite Rabs_mult.
199
198
replace r with (r*1) by auto with real.
200
199
apply Rmult_le_0_lt_compat;
You can’t perform that action at this time.
0 commit comments