Skip to content

Commit

Permalink
windRev
Browse files Browse the repository at this point in the history
  • Loading branch information
forked-from-1kasper committed Nov 4, 2023
1 parent afa7a09 commit d5eee8e
Showing 1 changed file with 10 additions and 4 deletions.
14 changes: 10 additions & 4 deletions GroundZero/HITs/Circle.lean
Original file line number Diff line number Diff line change
Expand Up @@ -139,15 +139,18 @@ namespace Circle
def base₁ : S¹ := Suspension.north
def base₂ : S¹ := Suspension.south

def seg₁ : base₁ = base₂ := Suspension.merid false
def seg₂ : base₁ = base₂ := Suspension.merid true
hott def seg₁ : base₁ = base₂ := Suspension.merid false
hott def seg₂ : base₁ = base₂ := Suspension.merid true

hott def ind₂ {B : S¹ → Type u} (b₁ : B base₁) (b₂ : B base₂)
(ℓ₁ : b₁ =[seg₁] b₂) (ℓ₂ : b₁ =[seg₂] b₂) : Π x, B x :=
Suspension.ind b₁ b₂ (λ | false => ℓ₁ | true => ℓ₂)

def base : S¹ := base₁
def loop : base = base := seg₂ ⬝ seg₁⁻¹
hott def base : S¹ := base₁
hott def loop : base = base := seg₂ ⬝ seg₁⁻¹

abbrev loop₁ : base₁ = base₁ := loop
hott def loop₂ : base₂ = base₂ := seg₁⁻¹ ⬝ seg₂

hott def rec {B : Type u} (b : B) (ℓ : b = b) : S¹ → B :=
Suspension.rec b b (λ | false => idp b | true => ℓ)
Expand Down Expand Up @@ -755,6 +758,9 @@ namespace Circle
symmetry; apply powerOfWinding; apply powerRev
end

noncomputable hott corollary windRev : Π {x : S¹} (p : x = x), wind x p⁻¹ = -(wind x p) :=
begin fapply indΩ; apply windingRev; intro; apply piProp; intro; apply Integer.set end

noncomputable hott lemma windingMult : Π (p q : Ω¹(S¹)), winding (mult p q) = winding p * winding q :=
begin
intro p; fapply Ωind₁;
Expand Down

0 comments on commit d5eee8e

Please sign in to comment.