Skip to content

Commit

Permalink
Update WeakTopology.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
yoh-tanimoto committed Mar 9, 2024
1 parent 7e23600 commit 49bf8ab
Showing 1 changed file with 31 additions and 7 deletions.
38 changes: 31 additions & 7 deletions WeakTopology/WeakTopology.lean
Original file line number Diff line number Diff line change
Expand Up @@ -40,14 +40,38 @@ theorem functional_convergence_of_norm_convergence


variable (x : E)
variable (z : WeakSpace π•œ E)
variable (n : β„•)
#check (x : WeakSpace π•œ E)
#check nhds (x : WeakSpace π•œ E)
#check nhds z
#check nhds n
#check nhds (n : ℝ)
#check (n : ℝ)
variable (z : WeakSpace π•œ E)
#check (z : E)


def Rdisc := TopCat.discrete.obj ℝ
lemma isDiscreteRdisc: DiscreteTopology (Rdisc) :=
⟨rfl⟩

variable (a : ℝ)
#check (a : Rdisc)
variable (b : Rdisc)
#check (b : ℝ)

variable (A : Set ℝ)
#check (A : Set Rdisc)
variable (B : Set Rdisc)
#check (B : Set ℝ)
def C := (A : Set Rdisc)
#check C A
#check (C A: Set ℝ)
#check IsOpen (C A)

#check isDiscreteRdisc

example : IsOpen B := by
exact (forall_open_iff_discrete.mpr isDiscreteRdisc) B

example : IsOpen (C A) := by
exact (forall_open_iff_discrete.mpr isDiscreteRdisc) (A : Set Rdisc)



variable (y : E β†’L[π•œ] π•œ)
variable (z : WeakDual π•œ E)
Expand Down

0 comments on commit 49bf8ab

Please sign in to comment.