File tree Expand file tree Collapse file tree 1 file changed +2
-10
lines changed Expand file tree Collapse file tree 1 file changed +2
-10
lines changed Original file line number Diff line number Diff line change @@ -108,22 +108,14 @@ section Preorder
108
108
109
109
variable [PartialOrder α] [Preorder β]
110
110
111
- -- porting note: type class search sees right through the type synonrm for `α ×ₗ β` and uses the
112
- -- `Preorder` structure for `α × β` instead
113
- -- This is hopefully the same problems as in https://github.com/leanprover/lean4/issues/1891
114
- -- and will be fixed in nightly-2022-11-30
115
- theorem toLex_mono : @Monotone _ _ _ (Prod.Lex.preorder α β) (toLex : α × β → α ×ₗ β) := by
111
+ theorem toLex_mono : Monotone (toLex : α × β → α ×ₗ β) := by
116
112
rintro ⟨a₁, b₁⟩ ⟨a₂, b₂⟩ ⟨ha, hb⟩
117
113
obtain rfl | ha : a₁ = a₂ ∨ _ := ha.eq_or_lt
118
114
· exact right _ hb
119
115
· exact left _ _ ha
120
116
#align prod.lex.to_lex_mono Prod.Lex.toLex_mono
121
117
122
- -- porting note: type class search sees right through the type synonrm for `α ×ₗ β` and uses the
123
- -- `Preorder` structure for `α × β` instead
124
- -- This is hopefully the same problems as in https://github.com/leanprover/lean4/issues/1891
125
- -- and will be fixed in nightly-2022-11-30
126
- theorem toLex_strictMono : @StrictMono _ _ _ (Prod.Lex.preorder α β) (toLex : α × β → α ×ₗ β) := by
118
+ theorem toLex_strictMono : StrictMono (toLex : α × β → α ×ₗ β) := by
127
119
rintro ⟨a₁, b₁⟩ ⟨a₂, b₂⟩ h
128
120
obtain rfl | ha : a₁ = a₂ ∨ _ := h.le.1 .eq_or_lt
129
121
· exact right _ (Prod.mk_lt_mk_iff_right.1 h)
You can’t perform that action at this time.
0 commit comments