Fixed Agda errors; fixed css errors which resulted in the incorrect font being used.

This commit is contained in:
Wen Kokke 2021-07-14 16:50:25 +01:00
parent edfb6c1601
commit 9691c05909
No known key found for this signature in database
GPG key ID: 7EB7DBBCEB539DB8
16 changed files with 19 additions and 18 deletions

View file

@ -12,7 +12,7 @@ TMP_DIR := $(CACHE_DIR)/tmp
################################################################################# #################################################################################
.PHONY: init .PHONY: init
init: setup-check-fix-whitespace setup-check-htmlproofer init: setup-check-fix-whitespace setup-install-htmlproofer
git config core.hooksPath .githooks git config core.hooksPath .githooks

View file

@ -982,9 +982,9 @@ Remember to indent all code by two spaces.
``` ```
ext∋ : ∀ {Γ B x y} ext∋ : ∀ {Γ B x y}
→ x ≢ y → x ≢ y
→ ¬ ∃[ A ]( Γ ∋ x ⦂ A ) → ¬ ( ∃[ A ] Γ ∋ x ⦂ A )
----------------------------- -----------------------------
→ ¬ ∃[ A ]( Γ , y ⦂ B ∋ x ⦂ A ) → ¬ ( ∃[ A ] Γ , y ⦂ B ∋ x ⦂ A )
ext∋ x≢y _ ⟨ A , Z ⟩ = x≢y refl ext∋ x≢y _ ⟨ A , Z ⟩ = x≢y refl
ext∋ _ ¬∃ ⟨ A , S _ ⊢x ⟩ = ¬∃ ⟨ A , ⊢x ⟩ ext∋ _ ¬∃ ⟨ A , S _ ⊢x ⟩ = ¬∃ ⟨ A , ⊢x ⟩
@ -1005,8 +1005,8 @@ Remember to indent all code by two spaces.
¬arg : ∀ {Γ A B L M} ¬arg : ∀ {Γ A B L M}
→ Γ ⊢ L ↑ A ⇒ B → Γ ⊢ L ↑ A ⇒ B
→ ¬ Γ ⊢ M ↓ A → ¬ Γ ⊢ M ↓ A
------------------------- ----------------------------
→ ¬ ∃[ B ](Γ ⊢ L · M ↑ B) → ¬ ( ∃[ B ] Γ ⊢ L · M ↑ B )
¬arg ⊢L ¬⊢M ⟨ B , ⊢L · ⊢M ⟩ rewrite dom≡ (uniq-↑ ⊢L ⊢L) = ¬⊢M ⊢M ¬arg ⊢L ¬⊢M ⟨ B , ⊢L · ⊢M ⟩ rewrite dom≡ (uniq-↑ ⊢L ⊢L) = ¬⊢M ⊢M
¬switch : ∀ {Γ M A B} ¬switch : ∀ {Γ M A B}

View file

@ -589,13 +589,14 @@ module Problem3 where
``` ```
ext∋ : ∀ {Γ B x y} ext∋ : ∀ {Γ B x y}
→ x ≢ y → x ≢ y
→ ¬ ∃[ A ]( Γ ∋ x ⦂ A ) → ¬ ( ∃[ A ] Γ ∋ x ⦂ A )
----------------------------- -----------------------------
→ ¬ ∃[ A ]( Γ , y ⦂ B ∋ x ⦂ A ) → ¬ ( ∃[ A ] Γ , y ⦂ B ∋ x ⦂ A )
ext∋ x≢y _ ⟨ A , Z ⟩ = x≢y refl ext∋ x≢y _ ⟨ A , Z ⟩ = x≢y refl
ext∋ _ ¬∃ ⟨ A , S _ ⊢x ⟩ = ¬∃ ⟨ A , ⊢x ⟩ ext∋ _ ¬∃ ⟨ A , S _ ⊢x ⟩ = ¬∃ ⟨ A , ⊢x ⟩
lookup : ∀ (Γ : Context) (x : Id) lookup :
∀ (Γ : Context) (x : Id)
----------------------- -----------------------
→ Dec (∃[ A ](Γ ∋ x ⦂ A)) → Dec (∃[ A ](Γ ∋ x ⦂ A))
lookup ∅ x = no (λ ()) lookup ∅ x = no (λ ())
@ -612,8 +613,8 @@ module Problem3 where
¬arg : ∀ {Γ A B L M} ¬arg : ∀ {Γ A B L M}
→ Γ ⊢ L ↑ A ⇒ B → Γ ⊢ L ↑ A ⇒ B
→ ¬ Γ ⊢ M ↓ A → ¬ Γ ⊢ M ↓ A
------------------------- ----------------------------
→ ¬ ∃[ B ](Γ ⊢ L · M ↑ B) → ¬ ( ∃[ B ] Γ ⊢ L · M ↑ B )
¬arg ⊢L ¬⊢M ⟨ B , ⊢L · ⊢M ⟩ rewrite dom≡ (uniq-↑ ⊢L ⊢L) = ¬⊢M ⊢M ¬arg ⊢L ¬⊢M ⟨ B , ⊢L · ⊢M ⟩ rewrite dom≡ (uniq-↑ ⊢L ⊢L) = ¬⊢M ⊢M
¬switch : ∀ {Γ M A B} ¬switch : ∀ {Γ M A B}

View file

@ -1,5 +1,5 @@
@import @import
"theme/skins/classic", "minima/skins/classic",
"theme/initialize", "minima/initialize",
"theme/agda" "minima/agda"
; ;

View file

@ -336,7 +336,7 @@ main = do
-- Compile CSS -- Compile CSS
match "css/*.css" $ compile compressCssCompiler match "css/*.css" $ compile compressCssCompiler
scss <- makePatternDependency "css/theme/**.scss" scss <- makePatternDependency "css/minima/**.scss"
rulesExtraDependencies [scss] $ rulesExtraDependencies [scss] $
match "css/minima.scss" $ match "css/minima.scss" $
compile $ sassCompilerWith sassOptions compile $ sassCompilerWith sassOptions

View file

@ -580,9 +580,9 @@ such that `Γ ∋ x ⦂ A` holds, then there is also no type `A` such that
``` ```
ext∋ : ∀ {Γ B x y} ext∋ : ∀ {Γ B x y}
→ x ≢ y → x ≢ y
→ ¬ ∃[ A ]( Γ ∋ x ⦂ A ) → ¬ ( ∃[ A ] Γ ∋ x ⦂ A )
----------------------------- -----------------------------
→ ¬ ∃[ A ]( Γ , y ⦂ B ∋ x ⦂ A ) → ¬ ( ∃[ A ] Γ , y ⦂ B ∋ x ⦂ A )
ext∋ x≢y _ ⟨ A , Z ⟩ = x≢y refl ext∋ x≢y _ ⟨ A , Z ⟩ = x≢y refl
ext∋ _ ¬∃ ⟨ A , S _ ∋x ⟩ = ¬∃ ⟨ A , ∋x ⟩ ext∋ _ ¬∃ ⟨ A , S _ ∋x ⟩ = ¬∃ ⟨ A , ∋x ⟩
``` ```
@ -638,8 +638,8 @@ there is no term `B` such that `Γ ⊢ L · M ↑ B` holds:
¬arg : ∀ {Γ A B L M} ¬arg : ∀ {Γ A B L M}
→ Γ ⊢ L ↑ A ⇒ B → Γ ⊢ L ↑ A ⇒ B
→ ¬ Γ ⊢ M ↓ A → ¬ Γ ⊢ M ↓ A
------------------------- ----------------------------
→ ¬ ∃[ B ](Γ ⊢ L · M ↑ B) → ¬ ( ∃[ B ] Γ ⊢ L · M ↑ B )
¬arg ⊢L ¬⊢M ⟨ B , ⊢L · ⊢M ⟩ rewrite dom≡ (uniq-↑ ⊢L ⊢L) = ¬⊢M ⊢M ¬arg ⊢L ¬⊢M ⟨ B , ⊢L · ⊢M ⟩ rewrite dom≡ (uniq-↑ ⊢L ⊢L) = ¬⊢M ⊢M
``` ```
Let `⊢L` be evidence that `Γ ⊢ L ↑ A ⇒ B` holds and `¬⊢M` be evidence Let `⊢L` be evidence that `Γ ⊢ L ↑ A ⇒ B` holds and `¬⊢M` be evidence