File tree Expand file tree Collapse file tree 3 files changed +522
-0
lines changed Expand file tree Collapse file tree 3 files changed +522
-0
lines changed Original file line number Diff line number Diff line change @@ -2218,6 +2218,8 @@ import Mathlib.Topology.Sets.Compacts
2218
2218
import Mathlib.Topology.Sets.Opens
2219
2219
import Mathlib.Topology.Sets.Order
2220
2220
import Mathlib.Topology.Sheaves.Abelian
2221
+ import Mathlib.Topology.Sheaves.Init
2222
+ import Mathlib.Topology.Sheaves.Presheaf
2221
2223
import Mathlib.Topology.ShrinkingLemma
2222
2224
import Mathlib.Topology.Sober
2223
2225
import Mathlib.Topology.Spectral.Hom
Original file line number Diff line number Diff line change
1
+ /-
2
+ Copyright (c) 2023 Jujian Zhang All rights reserved.
3
+ Released under Apache 2.0 license as described in the file LICENSE.
4
+ Authors: Jujian Zhang
5
+ -/
6
+
7
+ import Aesop
8
+
9
+ /-!
10
+ # Rule sets related to topological (pre)sheaves
11
+
12
+ This module defines the `Restrict` Aesop rule set. Aesop rule sets only become
13
+ visible once the file in which they're declared is imported, so we must put this
14
+ declaration into its own file.
15
+ -/
16
+
17
+ /- to prove subset relations -/
18
+ declare_aesop_rule_sets [Restrict]
You can’t perform that action at this time.
0 commit comments