File tree 1 file changed +10
-10
lines changed
1 file changed +10
-10
lines changed Original file line number Diff line number Diff line change @@ -502,15 +502,15 @@ variable [TopologicalSpace D] [IsActionTopology R D]
502
502
503
503
open scoped TensorProduct
504
504
505
- @[continuity, fun_prop]
506
- lemma continuous_mul : Continuous (fun ab ↦ ab.1 * ab.2 : D × D → D) := by
507
- letI : TopologicalSpace (D ⊗[R] D) := actionTopology R _
508
- haveI : IsActionTopology R (D ⊗[R] D) := { isActionTopology' := rfl }
509
- convert Module.continuous_bilinear_of_finite <| LinearMap.mul R D
510
-
511
- def Module.topologicalRing : TopologicalRing D where
512
- continuous_add := (isActionTopology_continuousAdd R D).1
513
- continuous_mul := continuous_mul R D
514
- continuous_neg := continuous_neg R D
505
+ -- @[continuity, fun_prop]
506
+ -- lemma continuous_mul : Continuous (fun ab ↦ ab.1 * ab.2 : D × D → D) := by
507
+ -- letI : TopologicalSpace (D ⊗[ R ] D) := actionTopology R _
508
+ -- haveI : IsActionTopology R (D ⊗[ R ] D) := { isActionTopology' := rfl }
509
+ -- convert Module.continuous_bilinear_of_finite <| LinearMap.mul R D
510
+
511
+ -- def Module.topologicalRing : TopologicalRing D where
512
+ -- continuous_add := (isActionTopology_continuousAdd R D).1
513
+ -- continuous_mul := continuous_mul' R D
514
+ -- continuous_neg := continuous_neg R D
515
515
516
516
end ring_algebra
You can’t perform that action at this time.
0 commit comments