File tree Expand file tree Collapse file tree 1 file changed +7
-0
lines changed Expand file tree Collapse file tree 1 file changed +7
-0
lines changed Original file line number Diff line number Diff line change @@ -54,6 +54,9 @@ protected def prod (f : Filter α) (g : Filter β) : Filter (α × β) :=
54
54
instance instSProd : SProd (Filter α) (Filter β) (Filter (α × β)) where
55
55
sprod := Filter.prod
56
56
57
+ theorem prod_eq_inf (f : Filter α) (g : Filter β) : f ×ˢ g = f.comap Prod.fst ⊓ g.comap Prod.snd :=
58
+ rfl
59
+
57
60
theorem prod_mem_prod (hs : s ∈ f) (ht : t ∈ g) : s ×ˢ t ∈ f ×ˢ g :=
58
61
inter_mem_inf (preimage_mem_comap hs) (preimage_mem_comap ht)
59
62
@@ -99,6 +102,10 @@ theorem comap_prod (f : α → β × γ) (b : Filter β) (c : Filter γ) :
99
102
comap f (b ×ˢ c) = comap (Prod.fst ∘ f) b ⊓ comap (Prod.snd ∘ f) c := by
100
103
erw [comap_inf, Filter.comap_comap, Filter.comap_comap]
101
104
105
+ theorem comap_prodMap_prod (f : α → β) (g : γ → δ) (lb : Filter β) (ld : Filter δ) :
106
+ comap (Prod.map f g) (lb ×ˢ ld) = comap f lb ×ˢ comap g ld := by
107
+ simp [prod_eq_inf, comap_comap, Function.comp_def]
108
+
102
109
theorem prod_top : f ×ˢ (⊤ : Filter β) = f.comap Prod.fst := by
103
110
dsimp only [SProd.sprod]
104
111
rw [Filter.prod, comap_top, inf_top_eq]
You can’t perform that action at this time.
0 commit comments