Skip to content

Commit

Permalink
add nix files to git ignore, update imports in tutorials
Browse files Browse the repository at this point in the history
  • Loading branch information
Peter Dragos authored and jespercockx committed Jun 9, 2024
1 parent 9388b77 commit 2d63a66
Show file tree
Hide file tree
Showing 3 changed files with 8 additions and 1 deletion.
4 changes: 4 additions & 0 deletions .gitignore
Original file line number Diff line number Diff line change
Expand Up @@ -7,3 +7,7 @@ docs/build/
*.hi
*.o

# For nix users
.direnv/**
.envrc
result
4 changes: 3 additions & 1 deletion tutorials/example-proofs/Ascending.agda
Original file line number Diff line number Diff line change
@@ -1,7 +1,9 @@
module Ascending where

open import Haskell.Prelude
open import Haskell.Prim
open import Haskell.Prim
open import Haskell.Law.Equality using (sym; begin_; _≡⟨⟩_; step-≡; _∎)
open import Haskell.Law.Bool using (ifTrueEqThen)

-- function judging ascending order on lists
isAscending : ⦃ iOrdA : Ord a ⦄ List a Bool
Expand Down
1 change: 1 addition & 0 deletions tutorials/example-proofs/Triangle.agda
Original file line number Diff line number Diff line change
@@ -1,6 +1,7 @@
module Triangle where

open import Haskell.Prelude
open import Haskell.Law.Bool using (&&-rightTrue; &&-leftTrue)

-- helper function
countBiggerThan : ⦃ Ord a ⦄ List a a Int
Expand Down

0 comments on commit 2d63a66

Please sign in to comment.