Skip to content

Commit 3cc0cb6

Browse files
committed
cleaning
1 parent f9729e8 commit 3cc0cb6

File tree

6 files changed

+8
-8
lines changed

6 files changed

+8
-8
lines changed

classical/classical_orders.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -329,7 +329,7 @@ Lemma big_lexi_order_interval_prefix (i : interval (big_lexi_order K))
329329
itv_open_ends i -> x \in i ->
330330
exists n, same_prefix n x `<=` [set` i].
331331
Proof.
332-
move: i; case=> [][[]l|[]] [[]r|[]] /orP []// ?; rewrite ?in_itv /= ?andbT.
332+
move: i; case=> [][[]l|[]] [[]r|[]]// ?; rewrite ?in_itv /= ?andbT.
333333
- move=> /andP[lx xr].
334334
case E1 : (first_diff l x) => [m|]; first last.
335335
by move: lx; move/first_diff_NoneP : E1 ->; rewrite bnd_simp.

classical/set_interval.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -868,8 +868,8 @@ End closed_endpoints.
868868
Lemma itv_open_endsI {d} {T : orderType d} (i j : interval T) :
869869
itv_open_ends i -> itv_open_ends j -> itv_open_ends (i `&` j)%O.
870870
Proof.
871-
move: i => [][[]a|[]] [[]b|[]] /orP []//= _;
872-
move: j => [][[]x|[]] [[]y|[]] /orP []//= _;
871+
move: i => [][[]a|[]] [[]b|[]]//=;
872+
move: j => [][[]x|[]] [[]y|[]]//=;
873873
by rewrite /itv_open_ends/= ?orbF ?andbT -?negb_or ?le_total//=;
874874
try ((by left)||(by right)).
875875
Qed.

theories/normedtype_theory/ereal_normedtype.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -496,7 +496,7 @@ apply/seteqP; split=> A.
496496
+ case=> M [Mreal MA].
497497
exists `]-oo, M%:E[ => [|y/=]; rewrite in_itv/= ?ltNyr; last exact: MA.
498498
by split => //; left.
499-
- move=> [[ [[]/= r|[]] [[]/= s|[]] ]] [] /orP []// _.
499+
- move=> [[ [[]/= r|[]] [[]/= s|[]] ]][]// _.
500500
+ move=> /[dup]/ltgte_fin_num/fineK <-; rewrite in_itv/=.
501501
move=> /andP[rx sx] rsA; apply: (nbhs_interval rx sx) => z rz zs.
502502
by apply: rsA =>/=; rewrite in_itv/= rz.

theories/topology_theory/num_topology.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -90,7 +90,7 @@ rewrite eqEsubset; split => U.
9090
by rewrite in_itv/= -lter_distl subrr normr0.
9191
apply: subset_trans xeU => z /=.
9292
by rewrite in_itv /= -lter_distl distrC.
93-
case => [][[[]l|[]]] [[]r|[]] [] /orP[]//= _.
93+
case => [][[[]l|[]]] [[]r|[]] []//= _.
9494
- move=> xlr lrU; exists (Order.min (x - l) (r - x)).
9595
by rewrite /= lt_min ?lterBDr ?add0r ?(itvP xlr).
9696
apply/(subset_trans _ lrU)/subset_ball_prop_in_itv.

theories/topology_theory/order_topology.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -95,7 +95,7 @@ Hint Resolve itv_open : core.
9595

9696
Lemma itv_open_ends_open (i : interval T) : itv_open_ends i -> open [set` i].
9797
Proof.
98-
case: i; rewrite /itv_open_ends => [[[]t1|[]]] [[]t2|[]] /orP[]? => //.
98+
case: i; rewrite /itv_open_ends => [[[]t1|[]]] [[]t2|[]]// ?.
9999
by rewrite set_itvE; exact: openT.
100100
Qed.
101101

@@ -225,7 +225,7 @@ pose j := \big[Order.meet/`]-oo, +oo[]_(i <- F) i.
225225
exists j; first split.
226226
- rewrite /j (@eq_fbig_cond _ _ _ _ _ F _ (mem F) _ id)//.
227227
+ apply: (big_ind itv_open_ends) => //=; first exact: itv_open_endsI.
228-
by rewrite /itv_open_ends; move=> i /rayF /set_mem ->.
228+
by rewrite /itv_open_ends; move=> i /rayF /set_mem ->.
229229
+ by move=> p /=; rewrite !inE/=; exact: andb_id2l.
230230
- pose f (i : interval T) : Prop := x \in i; suff : f j by [].
231231
rewrite /j (@eq_fbig_cond _ _ _ _ _ F _ (mem F) _ id)//=.

theories/topology_theory/weak_topology.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -203,7 +203,7 @@ Let WeakU : topologicalType := @weak_topology (sub_type Y) X val.
203203
Lemma open_order_weak (U : set Y) : @open OrdU U -> @open WeakU U.
204204
Proof.
205205
rewrite ?openE /= /interior => + x Ux => /(_ x Ux); rewrite itv_nbhsE /=.
206-
move=> [][][[]l|[]] [[]r|[]][]/orP[]//= _ xlr /filterS; apply.
206+
move=> [][][[]l|[]] [[]r|[]][]//= _ xlr /filterS; apply.
207207
- exists `]l, r[%classic; split => //=; exists `]\val l, \val r[%classic.
208208
exact: itv_open.
209209
by rewrite eqEsubset; split => z; rewrite preimage_itv.

0 commit comments

Comments
 (0)