Skip to content

Commit

Permalink
Check all agda files (#1058)
Browse files Browse the repository at this point in the history
* remove stuff with broken dependencies

* Revert "remove stuff with broken dependencies"

This reverts commit 6a0ded9.

* fix

* rm LocalizationDefs

* fixes/commented out lots of things

* no automatic Experiments/Everything.agda

* deleted the two files
  • Loading branch information
felixwellen authored Feb 2, 2024
1 parent 2ecfa00 commit c6a96ee
Show file tree
Hide file tree
Showing 11 changed files with 21 additions and 640 deletions.
1 change: 0 additions & 1 deletion .gitignore
Original file line number Diff line number Diff line change
Expand Up @@ -6,4 +6,3 @@ Cubical/*/Everything.agda
!Cubical/Core/Everything.agda
!Cubical/Foundations/Everything.agda
!Cubical/Codata/Everything.agda
!Cubical/Experiments/Everything.agda
3 changes: 2 additions & 1 deletion Cubical/Experiments/CohomologyGroups.agda
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
{-# OPTIONS --safe #-}
module Cubical.Experiments.CohomologyGroups where

{-
open import Cubical.Experiments.ZCohomologyOld.Base
open import Cubical.Experiments.ZCohomologyOld.Properties
open import Cubical.Experiments.ZCohomologyOld.MayerVietorisUnreduced
Expand Down Expand Up @@ -138,3 +138,4 @@ H¹-S¹≅ℤ =
Σ[ x ∈ Int ] (inv H⁰-S⁰≅ℤ×ℤ (x , x))
≡ GroupHom.fun (K.Δ 0) (∣ f ∣₂ , ∣ g ∣₂)
helper2 f g = (f _ -[ 0 ]ₖ g _) , cong ∣_∣₂ (funExt λ {true refl ; false refl})
-}
3 changes: 2 additions & 1 deletion Cubical/Experiments/Combinatorics.agda
Original file line number Diff line number Diff line change
Expand Up @@ -78,10 +78,11 @@ s = refl
p : prod (Fin _) f ≡ 6480
p = refl

{-
-- the maximal value
m : maxValue (Fin _) f ∣ fzero ∣ ≡ 9
m = refl

-}
-- the number of numeral 1
n1 : card (_ , isFinSetFiberDisc (Fin _) ℕ discreteℕ f 1) ≡ 2
n1 = refl
Expand Down
16 changes: 0 additions & 16 deletions Cubical/Experiments/Everything.agda

This file was deleted.

9 changes: 7 additions & 2 deletions Cubical/Experiments/HInt.agda
Original file line number Diff line number Diff line change
@@ -1,3 +1,4 @@
{-# OPTIONS --safe #-}
{-
Definition of the integers as a HIT inspired by slide 10 of (original
Expand All @@ -22,7 +23,8 @@ module Cubical.Experiments.HInt where
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Equiv
open import Cubical.Foundations.Isomorphism
open import Cubical.Data.Int

open import Cubical.Data.Int renaming (ℤ to Int; sucℤ to sucInt; predℤ to predInt; isSetℤ to isSetInt)
open import Cubical.Data.Nat

data : Type₀ where
Expand Down Expand Up @@ -77,22 +79,25 @@ lem2 (pos (suc n)) = sym (predsuc (ℕ→ℤ n))
lem2 (negsuc n) = refl

-- I don't see how to fill these holes, especially the last one
{-
ℤ→Int→ℤ : ∀ (n : ℤ) → Int→ℤ (ℤ→Int n) ≡ n
ℤ→Int→ℤ zero = refl
ℤ→Int→ℤ (suc n) = (lem1 (ℤ→Int n)) ∙ (cong suc (ℤ→Int→ℤ n))
ℤ→Int→ℤ (pred n) = (lem2 (ℤ→Int n)) ∙ (cong pred (ℤ→Int→ℤ n))
ℤ→Int→ℤ (sucpred n i) = {!!}
ℤ→Int→ℤ (predsuc n i) = {!!}
ℤ→Int→ℤ (coh n i j) = {!!}
-}

Int→ℤ→Int : n ℤ→Int (Int→ℤ n) ≡ n
Int→ℤ→Int (pos zero) = refl
Int→ℤ→Int (pos (suc n)) = cong sucInt (Int→ℤ→Int (pos n))
Int→ℤ→Int (negsuc zero) = refl
Int→ℤ→Int (negsuc (suc n)) = cong predInt (Int→ℤ→Int (negsuc n))

{-
Int≡ℤ : Int ≡ ℤ
Int≡ℤ = isoToPath (iso Int→ℤ ℤ→Int ℤ→Int→ℤ Int→ℤ→Int)
isSetℤ : isSet ℤ
isSetℤ = subst isSet Int≡ℤ isSetInt
-}
3 changes: 1 addition & 2 deletions Cubical/Experiments/IntegerMatrix.agda
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,6 @@ open import Cubical.Data.List

open import Cubical.Algebra.CommRing
open import Cubical.Algebra.CommRing.Instances.Int
renaming (ℤ to ℤRing)

open import Cubical.Algebra.Matrix
open import Cubical.Algebra.Matrix.CommRingCoefficient
Expand All @@ -27,7 +26,7 @@ private
variable
m n :

open Coefficient ℤRing
open Coefficient ℤCommRing

-- Get divisors directly

Expand Down
146 changes: 0 additions & 146 deletions Cubical/Experiments/LocalisationDefs.agda

This file was deleted.

79 changes: 0 additions & 79 deletions Cubical/Experiments/ZCohomologyExperiments.agda

This file was deleted.

Loading

0 comments on commit c6a96ee

Please sign in to comment.