@@ -262,60 +262,44 @@ end
262
262
263
263
end is_domain
264
264
265
- end sesq_form
266
-
267
- namespace refl_sesq_form
268
-
269
- open refl_sesq_form sesq_form
270
-
271
265
variables {R : Type *} {M : Type *} [ring R] [add_comm_group M] [module R M]
272
266
variables {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I}
273
267
274
268
/-- The proposition that a sesquilinear form is reflexive -/
275
269
def is_refl (S : sesq_form R M I) : Prop := ∀ (x y : M), S x y = 0 → S y x = 0
276
270
277
- variable (H : is_refl S)
278
-
279
- lemma eq_zero : ∀ {x y : M}, S x y = 0 → S y x = 0 := λ x y, H x y
280
-
281
- lemma ortho_sym {x y : M} :
282
- is_ortho S x y ↔ is_ortho S y x := ⟨eq_zero H, eq_zero H⟩
271
+ namespace is_refl
283
272
284
- end refl_sesq_form
273
+ variable (H : S.is_refl)
285
274
286
- namespace sym_sesq_form
275
+ lemma eq_zero : ∀ {x y : M}, S x y = 0 → S y x = 0 := λ x y, H x y
287
276
288
- open sym_sesq_form sesq_form
277
+ lemma ortho_comm {x y : M} : is_ortho S x y ↔ is_ortho S y x := ⟨eq_zero H, eq_zero H⟩
289
278
290
- variables {R : Type *} {M : Type *} [ring R] [add_comm_group M] [module R M]
291
- variables {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I}
279
+ end is_refl
292
280
293
281
/-- The proposition that a sesquilinear form is symmetric -/
294
- def is_sym (S : sesq_form R M I) : Prop := ∀ (x y : M), (I (S x y)).unop = S y x
295
-
296
- variable (H : is_sym S)
297
- include H
282
+ def is_symm (S : sesq_form R M I) : Prop := ∀ (x y : M), (I (S x y)).unop = S y x
298
283
299
- lemma sym (x y : M) : (I (S x y)).unop = S y x := H x y
284
+ namespace is_symm
300
285
301
- lemma is_refl : refl_sesq_form.is_refl S := λ x y H1, by { rw [←H], simp [H1], }
302
-
303
- lemma ortho_sym {x y : M} :
304
- is_ortho S x y ↔ is_ortho S y x := refl_sesq_form.ortho_sym (is_refl H)
286
+ variable (H : S.is_symm)
287
+ include H
305
288
306
- end sym_sesq_form
289
+ protected lemma eq (x y : M) : (I (S x y)).unop = S y x := H x y
307
290
308
- namespace alt_sesq_form
291
+ lemma is_refl : S.is_refl := λ x y H1, by { rw [←H], simp [H1], }
309
292
310
- open alt_sesq_form sesq_form
293
+ lemma ortho_comm {x y : M} : is_ortho S x y ↔ is_ortho S y x := H.is_refl.ortho_comm
311
294
312
- variables {R : Type *} {M : Type *} [ring R] [add_comm_group M] [module R M]
313
- variables {I : R ≃+* Rᵒᵖ} {S : sesq_form R M I}
295
+ end is_symm
314
296
315
297
/-- The proposition that a sesquilinear form is alternating -/
316
298
def is_alt (S : sesq_form R M I) : Prop := ∀ (x : M), S x x = 0
317
299
318
- variable (H : is_alt S)
300
+ namespace is_alt
301
+
302
+ variable (H : S.is_alt)
319
303
include H
320
304
321
305
lemma self_eq_zero (x : M) : S x x = 0 := H x
@@ -331,4 +315,14 @@ begin
331
315
exact H1,
332
316
end
333
317
334
- end alt_sesq_form
318
+ lemma is_refl : S.is_refl :=
319
+ begin
320
+ intros x y h,
321
+ rw [← neg H, h, neg_zero],
322
+ end
323
+
324
+ lemma ortho_comm {x y : M} : is_ortho S x y ↔ is_ortho S y x := H.is_refl.ortho_comm
325
+
326
+ end is_alt
327
+
328
+ end sesq_form
0 commit comments