Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 23cd34b

Browse files
committed
Revert "fix timeouts"
This reverts commit 933620c.
1 parent 933620c commit 23cd34b

File tree

1 file changed

+5
-16
lines changed

1 file changed

+5
-16
lines changed

src/topology/algebra/order/intermediate_value.lean

Lines changed: 5 additions & 16 deletions
Original file line numberDiff line numberDiff line change
@@ -386,10 +386,12 @@ begin
386386
exact (nhds_within_Ioi_self_ne_bot' ⟨b, hxab.2⟩).nonempty_of_mem this
387387
end
388388

389-
lemma is_preconnected_Icc_aux (x y : α) (s t : set α) (hxy : x ≤ y)
390-
(hs : is_closed s) (ht : is_closed t) (hab : Icc a b ⊆ s ∪ t)
391-
(hx : x ∈ Icc a b ∩ s) (hy : y ∈ Icc a b ∩ t) : (Icc a b ∩ (s ∩ t)).nonempty :=
389+
/-- A closed interval in a densely ordered conditionally complete linear order is preconnected. -/
390+
lemma is_preconnected_Icc : is_preconnected (Icc a b) :=
391+
is_preconnected_closed_iff.2
392392
begin
393+
rintros s t hs ht hab ⟨x, hx⟩ ⟨y, hy⟩,
394+
wlog hxy : x ≤ y := le_total x y using [x y s t, y x t s],
393395
have xyab : Icc x y ⊆ Icc a b := Icc_subset_Icc hx.1.1 hy.1.2,
394396
by_contradiction hst,
395397
suffices : Icc x y ⊆ s,
@@ -405,19 +407,6 @@ begin
405407
exact λ w ⟨wt, wzy⟩, (this wzy).elim id (λ h, (wt h).elim)
406408
end
407409

408-
/-- A closed interval in a densely ordered conditionally complete linear order is preconnected. -/
409-
lemma is_preconnected_Icc : is_preconnected (Icc a b) :=
410-
is_preconnected_closed_iff.2
411-
begin
412-
rintros s t hs ht hab ⟨x, hx⟩ ⟨y, hy⟩,
413-
-- This used to use `wlog`, but it was causing timeouts.
414-
cases le_total x y,
415-
{ exact is_preconnected_Icc_aux x y s t h hs ht hab hx hy, },
416-
{ rw inter_comm s t,
417-
rw union_comm s t at hab,
418-
exact is_preconnected_Icc_aux y x t s h ht hs hab hy hx, },
419-
end
420-
421410
lemma is_preconnected_interval : is_preconnected (interval a b) := is_preconnected_Icc
422411

423412
lemma set.ord_connected.is_preconnected {s : set α} (h : s.ord_connected) :

0 commit comments

Comments
 (0)