@@ -108,35 +108,15 @@ theorem numeric_neg : Π {x : pgame} (o : numeric x), numeric (-x)
108
108
⟨λ j i, lt_iff_neg_gt.1 (o.1 i j),
109
109
⟨λ j, numeric_neg (o.2 .2 j), λ i, numeric_neg (o.2 .1 i)⟩⟩
110
110
111
- -- We provide this as an analogue for `numeric.move_left_le`,
112
- -- even though it does not need the `numeric` hypothesis.
113
- @[nolint unused_arguments]
114
- theorem numeric.move_left_lt {x : pgame.{u}} (o : numeric x) (i : x.left_moves) :
115
- x.move_left i < x :=
116
- begin
117
- rw lt_def_le,
118
- left,
119
- use i,
120
- end
121
-
111
+ /-- For the `<` version, see `pgame.move_left_lt`. -/
122
112
theorem numeric.move_left_le {x : pgame} (o : numeric x) (i : x.left_moves) :
123
113
x.move_left i ≤ x :=
124
- le_of_lt (o.move_left i) o (o.move_left_lt i)
125
-
126
- -- We provide this as an analogue for `numeric.le_move_right`,
127
- -- even though it does not need the `numeric` hypothesis.
128
- @[nolint unused_arguments]
129
- theorem numeric.lt_move_right {x : pgame} (o : numeric x) (j : x.right_moves) :
130
- x < x.move_right j :=
131
- begin
132
- rw lt_def_le,
133
- right,
134
- use j,
135
- end
114
+ le_of_lt (o.move_left i) o (pgame.move_left_lt i)
136
115
116
+ /-- For the `<` version, see `pgame.lt_move_right`. -/
137
117
theorem numeric.le_move_right {x : pgame} (o : numeric x) (j : x.right_moves) :
138
118
x ≤ x.move_right j :=
139
- le_of_lt o (o.move_right j) (o .lt_move_right j)
119
+ le_of_lt o (o.move_right j) (pgame .lt_move_right j)
140
120
141
121
theorem add_lt_add
142
122
{w x y z : pgame.{u}} (oy : numeric y) (oz : numeric z)
@@ -178,10 +158,10 @@ theorem numeric_add : Π {x y : pgame} (ox : numeric x) (oy : numeric y), numeri
178
158
{ show xL ix + ⟨yl, yr, yL, yR⟩ < xR jx + ⟨yl, yr, yL, yR⟩,
179
159
exact add_lt_add_right (ox.1 ix jx) _ },
180
160
{ show xL ix + ⟨yl, yr, yL, yR⟩ < ⟨xl, xr, xL, xR⟩ + yR jy,
181
- exact add_lt_add oy (oy.move_right jy) (ox.move_left_lt _ ) (oy.lt_move_right _ ), },
182
- { -- show ⟨xl, xr, xL, xR⟩ + yL iy < xR jx + ⟨yl, yr, yL, yR⟩, -- fails?
183
- exact add_lt_add (oy.move_left iy) oy (ox.lt_move_right _ ) (oy.move_left_lt _ ), },
184
- { -- show ⟨xl, xr, xL, xR⟩ + yL iy < ⟨xl, xr, xL, xR⟩ + yR jy, -- fails?
161
+ exact add_lt_add oy (oy.move_right jy) (pgame.lt_mk ix ) (pgame.mk_lt jy ), },
162
+ { -- show ⟨xl, xr, xL, xR⟩ + yL iy < xR jx + ⟨yl, yr, yL, yR⟩, -- fails?
163
+ exact add_lt_add (oy.move_left iy) oy (pgame.mk_lt jx ) (pgame.lt_mk iy ), },
164
+ { -- show ⟨xl, xr, xL, xR⟩ + yL iy < ⟨xl, xr, xL, xR⟩ + yR jy, -- fails?
185
165
exact @add_lt_add_left pgame _ _ _ _ _ (oy.1 iy jy) ⟨xl, xr, xL, xR⟩ }
186
166
end ,
187
167
begin
0 commit comments