Skip to content

Commit 2f7863d

Browse files
chore: fix naming conventions in Order.WithBot (#801)
1 parent 932da6e commit 2f7863d

File tree

2 files changed

+61
-61
lines changed

2 files changed

+61
-61
lines changed

Mathlib/Order/RelClasses.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -792,7 +792,7 @@ theorem transitive_ge [Preorder α] : Transitive (@GE.ge α _) :=
792792
theorem transitive_gt [Preorder α] : Transitive (@GT.gt α _) :=
793793
transitive_of_trans _
794794

795-
instance OrderDual.is_total_le [LE α] [h : IsTotal α (· ≤ ·)] : IsTotal αᵒᵈ (· ≤ ·) :=
795+
instance OrderDual.isTotal_le [LE α] [h : IsTotal α (· ≤ ·)] : IsTotal αᵒᵈ (· ≤ ·) :=
796796
@IsTotal.swap α _ h
797797

798798
instance : WellFoundedLt ℕ :=

Mathlib/Order/WithBot.lean

Lines changed: 60 additions & 60 deletions
Original file line numberDiff line numberDiff line change
@@ -57,11 +57,11 @@ theorem coe_inj : (a : WithBot α) = b ↔ a = b :=
5757
Option.some_inj
5858
#align with_bot.coe_inj WithBot.coe_inj
5959

60-
protected theorem _root_.WithBot.forall {p : WithBot α → Prop} : (∀ x, p x) ↔ p ⊥ ∧ ∀ x : α, p x :=
60+
protected theorem «forall» {p : WithBot α → Prop} : (∀ x, p x) ↔ p ⊥ ∧ ∀ x : α, p x :=
6161
Option.forall
6262
#align with_bot.forall WithBot.forall
6363

64-
protected theorem _root_.WithBot.exists {p : WithBot α → Prop} : (∃ x, p x) ↔ p ⊥ ∨ ∃ x : α, p x :=
64+
protected theorem «exists» {p : WithBot α → Prop} : (∃ x, p x) ↔ p ⊥ ∨ ∃ x : α, p x :=
6565
Option.exists
6666
#align with_bot.exists WithBot.exists
6767

@@ -93,16 +93,16 @@ def recBotCoe {C : WithBot α → Sort _} (h₁ : C ⊥) (h₂ : ∀ a : α, C a
9393
#align with_bot.rec_bot_coe WithBot.recBotCoe
9494

9595
@[simp]
96-
theorem rec_bot_coe_bot {C : WithBot α → Sort _} (d : C ⊥) (f : ∀ a : α, C a) :
96+
theorem recBotCoe_bot {C : WithBot α → Sort _} (d : C ⊥) (f : ∀ a : α, C a) :
9797
@recBotCoe _ C d f ⊥ = d :=
9898
rfl
99-
#align with_bot.rec_bot_coe_bot WithBot.rec_bot_coe_bot
99+
#align with_bot.rec_bot_coe_bot WithBot.recBotCoe_bot
100100

101101
@[simp]
102-
theorem rec_bot_coe_coe {C : WithBot α → Sort _} (d : C ⊥) (f : ∀ a : α, C a) (x : α) :
102+
theorem recBotCoe_coe {C : WithBot α → Sort _} (d : C ⊥) (f : ∀ a : α, C a) (x : α) :
103103
@recBotCoe _ C d f ↑x = f x :=
104104
rfl
105-
#align with_bot.rec_bot_coe_coe WithBot.rec_bot_coe_coe
105+
#align with_bot.rec_bot_coe_coe WithBot.recBotCoe_coe
106106

107107
/-- Specialization of `option.get_or_else` to values in `with_bot α` that respects API boundaries.
108108
-/
@@ -295,9 +295,9 @@ instance [PartialOrder α] : PartialOrder (WithBot α) :=
295295
rw [le_antisymm h₁' h₂']
296296
}
297297

298-
theorem coe_strict_mono [Preorder α] : StrictMono (fun (a : α) => (a : WithBot α)) :=
298+
theorem coe_strictMono [Preorder α] : StrictMono (fun (a : α) => (a : WithBot α)) :=
299299
fun _ _ => coe_lt_coe.2
300-
#align with_bot.coe_strict_mono WithBot.coe_strict_mono
300+
#align with_bot.coe_strict_mono WithBot.coe_strictMono
301301

302302
theorem coe_mono [Preorder α] : Monotone (fun (a : α) => (a : WithBot α)) :=
303303
fun _ _ => coe_le_coe.2
@@ -320,21 +320,21 @@ theorem monotone_map_iff [Preorder α] [Preorder β] {f : α → β} :
320320

321321
alias monotone_map_iff ↔ _ _root_.monotone.with_bot_map
322322

323-
theorem strict_mono_iff [Preorder α] [Preorder β] {f : WithBot α → β} :
323+
theorem strictMono_iff [Preorder α] [Preorder β] {f : WithBot α → β} :
324324
StrictMono f ↔ StrictMono (λ a => f a : α → β) ∧ ∀ x : α, f ⊥ < f x :=
325-
fun h => ⟨h.comp WithBot.coe_strict_mono, fun _ => h (bot_lt_coe _)⟩, fun h =>
325+
fun h => ⟨h.comp WithBot.coe_strictMono, fun _ => h (bot_lt_coe _)⟩, fun h =>
326326
WithBot.forall.2
327327
⟨WithBot.forall.2 ⟨flip absurd (lt_irrefl _), fun x _ => h.2 x⟩, fun _ =>
328328
WithBot.forall.2fun h => (not_lt_bot h).elim, fun _ hle => h.1 (coe_lt_coe.1 hle)⟩⟩⟩
329-
#align with_bot.strict_mono_iff WithBot.strict_mono_iff
329+
#align with_bot.strict_mono_iff WithBot.strictMono_iff
330330

331331
@[simp]
332-
theorem strict_mono_map_iff [Preorder α] [Preorder β] {f : α → β} :
332+
theorem strictMono_map_iff [Preorder α] [Preorder β] {f : α → β} :
333333
StrictMono (WithBot.map f) ↔ StrictMono f :=
334-
strict_mono_iff.trans <| by simp [StrictMono, bot_lt_coe]
335-
#align with_bot.strict_mono_map_iff WithBot.strict_mono_map_iff
334+
strictMono_iff.trans <| by simp [StrictMono, bot_lt_coe]
335+
#align with_bot.strict_mono_map_iff WithBot.strictMono_map_iff
336336

337-
alias strict_mono_map_iff ↔ _ _root_.strict_mono.with_bot_map
337+
alias strictMono_map_iff ↔ _ _root_.StrictMono.with_bot_map
338338

339339
theorem map_le_iff [Preorder α] [Preorder β] (f : α → β) (mono_iff : ∀ {a b}, f a ≤ f b ↔ a ≤ b) :
340340
∀ a b : WithBot α, a.map f ≤ b.map f ↔ a ≤ b
@@ -416,27 +416,27 @@ instance [DistribLattice α] : DistribLattice (WithBot α) :=
416416
| (a₁ : α), (a₂ : α), ⊥ => inf_le_right
417417
| (a₁ : α), (a₂ : α), (a₃ : α) => coe_le_coe.mpr le_sup_inf }
418418

419-
instance decidableLe [LE α] [@DecidableRel α (· ≤ ·)] : @DecidableRel (WithBot α) (· ≤ ·)
419+
instance decidableLE [LE α] [@DecidableRel α (· ≤ ·)] : @DecidableRel (WithBot α) (· ≤ ·)
420420
| none, x => isTrue fun a h => Option.noConfusion h
421421
| Option.some x, Option.some y =>
422422
if h : x ≤ y then isTrue (some_le_some.2 h) else isFalse <| by simp [*]
423423
| Option.some x, none => isFalse fun h => by rcases h x rfl with ⟨y, ⟨_⟩, _⟩
424-
#align with_bot.decidable_le WithBot.decidableLe
424+
#align with_bot.decidable_le WithBot.decidableLE
425425

426-
instance decidableLt [LT α] [@DecidableRel α (· < ·)] : @DecidableRel (WithBot α) (· < ·)
426+
instance decidableLT [LT α] [@DecidableRel α (· < ·)] : @DecidableRel (WithBot α) (· < ·)
427427
| none, Option.some x => isTrue <| by exists x, rfl ; rintro _ ⟨⟩
428428
| Option.some x, Option.some y =>
429429
if h : x < y then isTrue <| by simp [*] else isFalse <| by simp [*]
430430
| x, none => isFalse <| by rintro ⟨a, ⟨⟨⟩⟩⟩
431-
#align with_bot.decidable_lt WithBot.decidableLt
431+
#align with_bot.decidable_lt WithBot.decidableLT
432432

433-
instance is_total_le [LE α] [IsTotal α (· ≤ ·)] : IsTotal (WithBot α) (· ≤ ·) :=
433+
instance isTotal_le [LE α] [IsTotal α (· ≤ ·)] : IsTotal (WithBot α) (· ≤ ·) :=
434434
fun a b =>
435435
match a, b with
436436
| none, _ => Or.inl bot_le
437437
| _, none => Or.inr bot_le
438438
| Option.some x, Option.some y => (total_of (· ≤ ·) x y).imp some_le_some.2 some_le_some.2
439-
#align with_bot.is_total_le WithBot.is_total_le
439+
#align with_bot.is_total_le WithBot.isTotal_le
440440

441441
instance [LinearOrder α] : LinearOrder (WithBot α) :=
442442
Lattice.toLinearOrder _
@@ -453,7 +453,7 @@ theorem coe_max [LinearOrder α] (x y : α) : ((max x y : α) : WithBot α) = ma
453453
rfl
454454
#align with_bot.coe_max WithBot.coe_max
455455

456-
theorem well_founded_lt [Preorder α] (h : @WellFounded α (· < ·)) :
456+
theorem wellFounded_lt [Preorder α] (h : @WellFounded α (· < ·)) :
457457
@WellFounded (WithBot α) (· < ·) :=
458458
have acc_bot : Acc ((· < ·) : WithBot α → WithBot α → Prop) ⊥ :=
459459
Acc.intro _ fun _ ha => (not_le_of_gt ha bot_le).elim
@@ -471,7 +471,7 @@ theorem well_founded_lt [Preorder α] (h : @WellFounded α (· < ·)) :
471471
Acc.intro _ fun c =>
472472
Option.recOn c (fun _ => acc_bot) fun _ hc => ih _
473473
(some_lt_some.1 hc) (lt_trans hc hba))⟩
474-
#align with_bot.well_founded_lt WithBot.well_founded_lt
474+
#align with_bot.well_founded_lt WithBot.wellFounded_lt
475475

476476
instance [LT α] [DenselyOrdered α] [NoMinOrder α] : DenselyOrdered (WithBot α) :=
477477
fun a b =>
@@ -545,11 +545,11 @@ instance : Top (WithTop α) :=
545545
instance : Inhabited (WithTop α) :=
546546
⟨⊤⟩
547547

548-
protected theorem _root_.WithTop.forall {p : WithTop α → Prop} : (∀ x, p x) ↔ p ⊤ ∧ ∀ x : α, p x :=
548+
protected theorem «forall» {p : WithTop α → Prop} : (∀ x, p x) ↔ p ⊤ ∧ ∀ x : α, p x :=
549549
Option.forall
550550
#align with_top.forall WithTop.forall
551551

552-
protected theorem _root_.WithTop.exists {p : WithTop α → Prop} : (∃ x, p x) ↔ p ⊤ ∨ ∃ x : α, p x :=
552+
protected theorem «exists» {p : WithTop α → Prop} : (∃ x, p x) ↔ p ⊤ ∨ ∃ x : α, p x :=
553553
Option.exists
554554
#align with_top.exists WithTop.exists
555555

@@ -579,16 +579,16 @@ def recTopCoe {C : WithTop α → Sort _} (h₁ : C ⊤) (h₂ : ∀ a : α, C a
579579
#align with_top.rec_top_coe WithTop.recTopCoe
580580

581581
@[simp]
582-
theorem rec_top_coe_top {C : WithTop α → Sort _} (d : C ⊤) (f : ∀ a : α, C a) :
582+
theorem recTopCoe_top {C : WithTop α → Sort _} (d : C ⊤) (f : ∀ a : α, C a) :
583583
@recTopCoe _ C d f ⊤ = d :=
584584
rfl
585-
#align with_top.rec_top_coe_top WithTop.rec_top_coe_top
585+
#align with_top.rec_top_coe_top WithTop.recTopCoe_top
586586

587587
@[simp]
588-
theorem rec_top_coe_coe {C : WithTop α → Sort _} (d : C ⊤) (f : ∀ a : α, C a) (x : α) :
588+
theorem recTopCoe_coe {C : WithTop α → Sort _} (d : C ⊤) (f : ∀ a : α, C a) (x : α) :
589589
@recTopCoe _ C d f ↑x = f x :=
590590
rfl
591-
#align with_top.rec_top_coe_coe WithTop.rec_top_coe_coe
591+
#align with_top.rec_top_coe_coe WithTop.recTopCoe_coe
592592

593593
/-- `WithTop.toDual` is the equivalence sending `⊤` to `⊥` and any `a : α` to `toDual a : αᵒᵈ`.
594594
See `WithTop.toDualBotEquiv` for the related order-iso.
@@ -1045,9 +1045,9 @@ instance [PartialOrder α] : PartialOrder (WithTop α) :=
10451045
simp_rw [← toDual_le_toDual_iff]
10461046
exact Function.swap le_antisymm }
10471047

1048-
theorem coe_strict_mono [Preorder α] : StrictMono (fun a : α => (a : WithTop α)) :=
1048+
theorem coe_strictMono [Preorder α] : StrictMono (fun a : α => (a : WithTop α)) :=
10491049
fun _ _ => some_lt_some.2
1050-
#align with_top.coe_strict_mono WithTop.coe_strict_mono
1050+
#align with_top.coe_strict_mono WithTop.coe_strictMono
10511051

10521052
theorem coe_mono [Preorder α] : Monotone (fun a : α => (a : WithTop α)) :=
10531053
fun _ _ => coe_le_coe.2
@@ -1069,21 +1069,21 @@ theorem monotone_map_iff [Preorder α] [Preorder β] {f : α → β} :
10691069

10701070
alias monotone_map_iff ↔ _ _root_.monotone.with_top_map
10711071

1072-
theorem strict_mono_iff [Preorder α] [Preorder β] {f : WithTop α → β} :
1072+
theorem strictMono_iff [Preorder α] [Preorder β] {f : WithTop α → β} :
10731073
StrictMono f ↔ StrictMono (fun (a : α) => f a) ∧ ∀ x : α, f x < f ⊤ :=
1074-
fun h => ⟨h.comp WithTop.coe_strict_mono, fun _ => h (coe_lt_top _)⟩, fun h =>
1074+
fun h => ⟨h.comp WithTop.coe_strictMono, fun _ => h (coe_lt_top _)⟩, fun h =>
10751075
WithTop.forall.2
10761076
⟨WithTop.forall.2 ⟨flip absurd (lt_irrefl _), fun _ h => (not_top_lt h).elim⟩, fun x =>
10771077
WithTop.forall.2fun _ => h.2 x, fun _ hle => h.1 (coe_lt_coe.1 hle)⟩⟩⟩
1078-
#align with_top.strict_mono_iff WithTop.strict_mono_iff
1078+
#align with_top.strict_mono_iff WithTop.strictMono_iff
10791079

10801080
@[simp]
1081-
theorem strict_mono_map_iff [Preorder α] [Preorder β] {f : α → β} :
1081+
theorem strictMono_map_iff [Preorder α] [Preorder β] {f : α → β} :
10821082
StrictMono (WithTop.map f) ↔ StrictMono f :=
1083-
strict_mono_iff.trans <| by simp [StrictMono, coe_lt_top]
1084-
#align with_top.strict_mono_map_iff WithTop.strict_mono_map_iff
1083+
strictMono_iff.trans <| by simp [StrictMono, coe_lt_top]
1084+
#align with_top.strict_mono_map_iff WithTop.strictMono_map_iff
10851085

1086-
alias strict_mono_map_iff ↔ _ _root_.strict_mono.with_top_map
1086+
alias strictMono_map_iff ↔ _ _root_.StrictMono.with_top_map
10871087

10881088
theorem map_le_iff [Preorder α] [Preorder β] (f : α → β) (a b : WithTop α)
10891089
(mono_iff : ∀ {a b}, f a ≤ f b ↔ a ≤ b) :
@@ -1156,11 +1156,11 @@ instance decidableLt [LT α] [@DecidableRel α (· < ·)] :
11561156
decidable_of_decidable_of_iff toDual_lt_toDual_iff
11571157
#align with_top.decidable_lt WithTop.decidableLt
11581158

1159-
instance is_total_le [LE α] [IsTotal α (· ≤ ·)] : IsTotal (WithTop α) (· ≤ ·) :=
1159+
instance isTotal_le [LE α] [IsTotal α (· ≤ ·)] : IsTotal (WithTop α) (· ≤ ·) :=
11601160
fun _ _ => by
11611161
simp_rw [← toDual_le_toDual_iff]
11621162
exact total_of _ _ _⟩
1163-
#align with_top.is_total_le WithTop.is_total_le
1163+
#align with_top.is_total_le WithTop.isTotal_le
11641164

11651165
instance [LinearOrder α] : LinearOrder (WithTop α) :=
11661166
Lattice.toLinearOrder _
@@ -1175,7 +1175,7 @@ theorem coe_max [LinearOrder α] (x y : α) : (↑(max x y) : WithTop α) = max
11751175
rfl
11761176
#align with_top.coe_max WithTop.coe_max
11771177

1178-
theorem well_founded_lt [Preorder α] (h : @WellFounded α (· < ·)) :
1178+
theorem wellFounded_lt [Preorder α] (h : @WellFounded α (· < ·)) :
11791179
@WellFounded (WithTop α) (· < ·) :=
11801180
have acc_some : ∀ a : α, Acc ((· < ·) : WithTop α → WithTop α → Prop) (some a) := fun a =>
11811181
Acc.intro _
@@ -1189,15 +1189,15 @@ theorem well_founded_lt [Preorder α] (h : @WellFounded α (· < ·)) :
11891189
fun a =>
11901190
Option.recOn a (Acc.intro _ fun y => Option.recOn y
11911191
(fun h => (lt_irrefl _ h).elim) fun _ _ => acc_some _) acc_some⟩
1192-
#align with_top.well_founded_lt WithTop.well_founded_lt
1192+
#align with_top.well_founded_lt WithTop.wellFounded_lt
11931193

11941194
open OrderDual
11951195

1196-
theorem well_founded_gt [Preorder α] (h : @WellFounded α (· > ·)) :
1196+
theorem wellFounded_gt [Preorder α] (h : @WellFounded α (· > ·)) :
11971197
@WellFounded (WithTop α) (· > ·) :=
11981198
fun a => by
11991199
-- ideally, use rel_hom_class.acc, but that is defined later
1200-
have : Acc (· < ·) (WithTop.toDual a) := WellFounded.apply (WithBot.well_founded_lt
1200+
have : Acc (· < ·) (WithTop.toDual a) := WellFounded.apply (WithBot.wellFounded_lt
12011201
(by convert h)) _
12021202
revert this
12031203
generalize ha : WithBot.toDual a = b
@@ -1206,70 +1206,70 @@ theorem well_founded_gt [Preorder α] (h : @WellFounded α (· > ·)) :
12061206
induction' ac with _ H IH generalizing a
12071207
subst ha
12081208
exact ⟨_, fun a' h => IH (WithTop.toDual a') (toDual_lt_toDual.mpr h) _ rfl⟩⟩
1209-
#align with_top.well_founded_gt WithTop.well_founded_gt
1209+
#align with_top.well_founded_gt WithTop.wellFounded_gt
12101210

1211-
theorem _root_.WithBot.well_founded_gt [Preorder α] (h : @WellFounded α (· > ·)) :
1211+
theorem _root_.WithBot.wellFounded_gt [Preorder α] (h : @WellFounded α (· > ·)) :
12121212
@WellFounded (WithBot α) (· > ·) :=
12131213
fun a => by
12141214
-- ideally, use rel_hom_class.acc, but that is defined later
12151215
have : Acc (· < ·) (WithBot.toDual a) :=
1216-
WellFounded.apply (WithTop.well_founded_lt (by convert h)) _
1216+
WellFounded.apply (WithTop.wellFounded_lt (by convert h)) _
12171217
revert this
12181218
generalize ha : WithBot.toDual a = b
12191219
intro ac
12201220
dsimp at ac
12211221
induction' ac with _ H IH generalizing a
12221222
subst ha
12231223
exact ⟨_, fun a' h => IH (WithBot.toDual a') (toDual_lt_toDual.mpr h) _ rfl⟩⟩
1224-
#align with_bot.well_founded_gt WithBot.well_founded_gt
1224+
#align with_bot.well_founded_gt WithBot.wellFounded_gt
12251225

1226-
instance Trichotomous.lt [Preorder α] [IsTrichotomous α (· < ·)] :
1226+
instance trichotomous.lt [Preorder α] [IsTrichotomous α (· < ·)] :
12271227
IsTrichotomous (WithTop α) (· < ·) :=
12281228
by
12291229
rintro (a | a) (b | b)
12301230
. simp
12311231
. simp
12321232
. simp
12331233
. simpa [some_eq_coe, IsTrichotomous, coe_eq_coe] using @trichotomous α (. < .) _ a b⟩
1234-
#align with_top.trichotomous.lt WithTop.Trichotomous.lt
1234+
#align with_top.trichotomous.lt WithTop.trichotomous.lt
12351235

12361236
instance IsWellOrder.lt [Preorder α] [h : IsWellOrder α (· < ·)] :
1237-
IsWellOrder (WithTop α) (· < ·) where wf := well_founded_lt h.wf
1237+
IsWellOrder (WithTop α) (· < ·) where wf := wellFounded_lt h.wf
12381238
#align with_top.is_well_order.lt WithTop.IsWellOrder.lt
12391239

1240-
instance Trichotomous.gt [Preorder α] [IsTrichotomous α (· > ·)] :
1240+
instance trichotomous.gt [Preorder α] [IsTrichotomous α (· > ·)] :
12411241
IsTrichotomous (WithTop α) (· > ·) :=
12421242
by
12431243
rintro (a | a) (b | b)
12441244
. simp
12451245
. simp
12461246
. simp
12471247
. simpa [some_eq_coe, IsTrichotomous, coe_eq_coe] using @trichotomous α (. > .) _ a b⟩
1248-
#align with_top.trichotomous.gt WithTop.Trichotomous.gt
1248+
#align with_top.trichotomous.gt WithTop.trichotomous.gt
12491249

12501250
instance IsWellOrder.gt [Preorder α] [h : IsWellOrder α (· > ·)] :
1251-
IsWellOrder (WithTop α) (· > ·) where wf := well_founded_gt h.wf
1251+
IsWellOrder (WithTop α) (· > ·) where wf := wellFounded_gt h.wf
12521252
#align with_top.is_well_order.gt WithTop.IsWellOrder.gt
12531253

12541254
instance _root_.WithBot.trichotomous.lt [Preorder α] [h : IsTrichotomous α (· < ·)] :
12551255
IsTrichotomous (WithBot α) (· < ·) :=
1256-
@WithTop.Trichotomous.gt αᵒᵈ _ h
1256+
@WithTop.trichotomous.gt αᵒᵈ _ h
12571257
#align with_bot.trichotomous.lt WithBot.trichotomous.lt
12581258

1259-
instance _root_.WithBot.is_well_order.lt [Preorder α] [h : IsWellOrder α (· < ·)] :
1259+
instance _root_.WithBot.isWellOrder.lt [Preorder α] [h : IsWellOrder α (· < ·)] :
12601260
IsWellOrder (WithBot α) (· < ·) :=
12611261
@WithTop.IsWellOrder.gt αᵒᵈ _ h
1262-
#align with_bot.is_well_order.lt WithBot.is_well_order.lt
1262+
#align with_bot.is_well_order.lt WithBot.isWellOrder.lt
12631263

12641264
instance _root_.WithBot.trichotomous.gt [Preorder α] [h : IsTrichotomous α (· > ·)] :
12651265
IsTrichotomous (WithBot α) (· > ·) :=
1266-
@WithTop.Trichotomous.lt αᵒᵈ _ h
1266+
@WithTop.trichotomous.lt αᵒᵈ _ h
12671267
#align with_bot.trichotomous.gt WithBot.trichotomous.gt
12681268

1269-
instance _root_.WithBot.is_well_order.gt [Preorder α] [h : IsWellOrder α (· > ·)] :
1269+
instance _root_.WithBot.isWellOrder.gt [Preorder α] [h : IsWellOrder α (· > ·)] :
12701270
IsWellOrder (WithBot α) (· > ·) :=
12711271
@WithTop.IsWellOrder.lt αᵒᵈ _ h
1272-
#align with_top._root_.with_bot.is_well_order.gt WithBot.is_well_order.gt
1272+
#align with_top._root_.with_bot.is_well_order.gt WithBot.isWellOrder.gt
12731273

12741274
instance [LT α] [DenselyOrdered α] [NoMaxOrder α] : DenselyOrdered (WithTop α) :=
12751275
instDenselyOrderedOrderDualInstLTOrderDual (WithBot αᵒᵈ)

0 commit comments

Comments
 (0)