Skip to content

Commit c0be162

Browse files
urkudmo271int-y1jjaassoonn
committed
feat: port Topology.Sheaves.Presheaf (#3828)
Co-authored-by: Moritz Firsching <firsching@google.com> Co-authored-by: int-y1 <jason_yuen2007@hotmail.com> Co-authored-by: Jujian Zhang <jujian.zhang1998@outlook.com>
1 parent ee5111f commit c0be162

File tree

3 files changed

+522
-0
lines changed

3 files changed

+522
-0
lines changed

Mathlib.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -2218,6 +2218,8 @@ import Mathlib.Topology.Sets.Compacts
22182218
import Mathlib.Topology.Sets.Opens
22192219
import Mathlib.Topology.Sets.Order
22202220
import Mathlib.Topology.Sheaves.Abelian
2221+
import Mathlib.Topology.Sheaves.Init
2222+
import Mathlib.Topology.Sheaves.Presheaf
22212223
import Mathlib.Topology.ShrinkingLemma
22222224
import Mathlib.Topology.Sober
22232225
import Mathlib.Topology.Spectral.Hom

Mathlib/Topology/Sheaves/Init.lean

Lines changed: 18 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,18 @@
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]

0 commit comments

Comments
 (0)