geometry.manifold.sheaf.basicMathlib.Geometry.Manifold.Sheaf.Basic

This file has been ported!

Changes since the initial port

The following section lists changes to this file in mathlib3 and mathlib4 that occured after the initial port. Most recent changes are shown first. Hovering over a commit will show all commits associated with the same mathlib3 commit.

Changes in mathlib3

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(last sync)

Changes in mathlib3port

mathlib3
mathlib3port
Diff
@@ -3,8 +3,8 @@ Copyright © 2023 Heather Macbeth. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Heather Macbeth
 -/
-import Mathbin.Geometry.Manifold.LocalInvariantProperties
-import Mathbin.Topology.Sheaves.LocalPredicate
+import Geometry.Manifold.LocalInvariantProperties
+import Topology.Sheaves.LocalPredicate
 
 #align_import geometry.manifold.sheaf.basic from "leanprover-community/mathlib"@"fdc286cc6967a012f41b87f76dcd2797b53152af"
 
Diff
@@ -2,15 +2,12 @@
 Copyright © 2023 Heather Macbeth. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Heather Macbeth
-
-! This file was ported from Lean 3 source module geometry.manifold.sheaf.basic
-! leanprover-community/mathlib commit fdc286cc6967a012f41b87f76dcd2797b53152af
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathbin.Geometry.Manifold.LocalInvariantProperties
 import Mathbin.Topology.Sheaves.LocalPredicate
 
+#align_import geometry.manifold.sheaf.basic from "leanprover-community/mathlib"@"fdc286cc6967a012f41b87f76dcd2797b53152af"
+
 /-! # Generic construction of a sheaf from a `local_invariant_prop` on a manifold
 
 > THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
Diff
@@ -96,7 +96,7 @@ a sheaf of types on `M` which, to each open set `U` in `M`, associates the type
 functions from `U` to `M'` satisfying the lift of `P`. -/
 def StructureGroupoid.LocalInvariantProp.sheaf (hG : LocalInvariantProp G G' P) :
     TopCat.Sheaf (Type u) (TopCat.of M) :=
-  TopCat.subsheafToTypes (hG.LocalPredicateₓ M M')
+  TopCat.subsheafToTypes (hG.LocalPredicate M M')
 #align structure_groupoid.local_invariant_prop.sheaf StructureGroupoid.LocalInvariantProp.sheaf
 -/
 
Diff
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Heather Macbeth
 
 ! This file was ported from Lean 3 source module geometry.manifold.sheaf.basic
-! leanprover-community/mathlib commit 431589bce478b2229eba14b14a283250428217db
+! leanprover-community/mathlib commit fdc286cc6967a012f41b87f76dcd2797b53152af
 ! Please do not edit these lines, except to modify the commit id
 ! if you have ported upstream changes.
 -/
@@ -13,6 +13,9 @@ import Mathbin.Topology.Sheaves.LocalPredicate
 
 /-! # Generic construction of a sheaf from a `local_invariant_prop` on a manifold
 
+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> Any changes to this file require a corresponding PR to mathlib4.
+
 This file constructs the sheaf-of-types of functions `f : M → M'` (for charted spaces `M`, `M'`)
 which satisfy the lifted property `lift_prop P` associated to some locally invariant (in the sense
 of `structure_groupoid.local_invariant_prop`) property `P` on the model spaces of `M` and `M'`. For
Diff
@@ -45,14 +45,19 @@ variable {H : Type _} [TopologicalSpace H] {H' : Type _} [TopologicalSpace H']
   (M : Type u) [TopologicalSpace M] [ChartedSpace H M] (M' : Type u) [TopologicalSpace M']
   [ChartedSpace H' M']
 
+#print TopCat.of.chartedSpace /-
 instance TopCat.of.chartedSpace : ChartedSpace H (TopCat.of M) :=
   (inferInstance : ChartedSpace H M)
 #align Top.of.charted_space TopCat.of.chartedSpace
+-/
 
+#print TopCat.of.hasGroupoid /-
 instance TopCat.of.hasGroupoid [HasGroupoid M G] : HasGroupoid (TopCat.of M) G :=
   (inferInstance : HasGroupoid M G)
 #align Top.of.has_groupoid TopCat.of.hasGroupoid
+-/
 
+#print StructureGroupoid.LocalInvariantProp.localPredicate /-
 /-- Let `P` be a `local_invariant_prop` for functions between spaces with the groupoids `G`, `G'`
 and let `M`, `M'` be charted spaces modelled on the model spaces of those groupoids.  Then there is
 an induced `local_predicate` on the functions from `M` to `M'`, given by `lift_prop P`. -/
@@ -79,7 +84,9 @@ def StructureGroupoid.LocalInvariantProp.localPredicate (hG : LocalInvariantProp
     ext1
     rfl
 #align structure_groupoid.local_invariant_prop.local_predicate StructureGroupoid.LocalInvariantProp.localPredicate
+-/
 
+#print StructureGroupoid.LocalInvariantProp.sheaf /-
 /-- Let `P` be a `local_invariant_prop` for functions between spaces with the groupoids `G`, `G'`
 and let `M`, `M'` be charted spaces modelled on the model spaces of those groupoids.  Then there is
 a sheaf of types on `M` which, to each open set `U` in `M`, associates the type of bundled
@@ -88,14 +95,19 @@ def StructureGroupoid.LocalInvariantProp.sheaf (hG : LocalInvariantProp G G' P)
     TopCat.Sheaf (Type u) (TopCat.of M) :=
   TopCat.subsheafToTypes (hG.LocalPredicateₓ M M')
 #align structure_groupoid.local_invariant_prop.sheaf StructureGroupoid.LocalInvariantProp.sheaf
+-/
 
+#print StructureGroupoid.LocalInvariantProp.sheafHasCoeToFun /-
 instance StructureGroupoid.LocalInvariantProp.sheafHasCoeToFun (hG : LocalInvariantProp G G' P)
     (U : (Opens (TopCat.of M))ᵒᵖ) : CoeFun ((hG.Sheaf M M').val.obj U) fun _ => unop U → M'
     where coe a := a.1
 #align structure_groupoid.local_invariant_prop.sheaf_has_coe_to_fun StructureGroupoid.LocalInvariantProp.sheafHasCoeToFun
+-/
 
+#print StructureGroupoid.LocalInvariantProp.section_spec /-
 theorem StructureGroupoid.LocalInvariantProp.section_spec (hG : LocalInvariantProp G G' P)
     (U : (Opens (TopCat.of M))ᵒᵖ) (f : (hG.Sheaf M M').val.obj U) : LiftProp P f :=
   f.2
 #align structure_groupoid.local_invariant_prop.section_spec StructureGroupoid.LocalInvariantProp.section_spec
+-/
 

Changes in mathlib4

mathlib3
mathlib4
chore: banish Type _ and Sort _ (#6499)

We remove all possible occurences of Type _ and Sort _ in favor of Type* and Sort*.

This has nice performance benefits.

Diff
@@ -37,7 +37,7 @@ open Set TopologicalSpace StructureGroupoid StructureGroupoid.LocalInvariantProp
 
 universe u
 
-variable {H : Type _} [TopologicalSpace H] {H' : Type _} [TopologicalSpace H']
+variable {H : Type*} [TopologicalSpace H] {H' : Type*} [TopologicalSpace H']
   {G : StructureGroupoid H} {G' : StructureGroupoid H'} {P : (H → H') → Set H → H → Prop}
   (M : Type u) [TopologicalSpace M] [ChartedSpace H M] (M' : Type u) [TopologicalSpace M']
   [ChartedSpace H' M']
chore: script to replace headers with #align_import statements (#5979)

Open in Gitpod

Co-authored-by: Eric Wieser <wieser.eric@gmail.com> Co-authored-by: Scott Morrison <scott.morrison@gmail.com>

Diff
@@ -2,15 +2,12 @@
 Copyright © 2023 Heather Macbeth. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Heather Macbeth
-
-! This file was ported from Lean 3 source module geometry.manifold.sheaf.basic
-! leanprover-community/mathlib commit 431589bce478b2229eba14b14a283250428217db
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathlib.Geometry.Manifold.LocalInvariantProperties
 import Mathlib.Topology.Sheaves.LocalPredicate
 
+#align_import geometry.manifold.sheaf.basic from "leanprover-community/mathlib"@"431589bce478b2229eba14b14a283250428217db"
+
 /-! # Generic construction of a sheaf from a `LocalInvariantProp` on a manifold
 
 This file constructs the sheaf-of-types of functions `f : M → M'` (for charted spaces `M`, `M'`)
feat: port Geometry.Manifold.Sheaf.Basic (#5373)

Dependencies 11 + 832

833 files ported (98.7%)
347704 lines ported (98.5%)
Show graph

The unported dependencies are