feat: part 8-2
This commit is contained in:
parent
b10afe5239
commit
68a806b291
|
@ -15,3 +15,4 @@ import public Day6.Part2
|
|||
import public Day7.Part1
|
||||
import public Day7.Part2
|
||||
import public Day8.Part1
|
||||
import public Day8.Part2
|
||||
|
|
|
@ -9,11 +9,13 @@ import Utils
|
|||
|
||||
--- TYPES
|
||||
|
||||
public export
|
||||
Map : (h, w : Nat) -> Type
|
||||
Map h w = Grid h w (Maybe Char)
|
||||
|
||||
--- PARSING
|
||||
|
||||
export
|
||||
parseInput : String -> Maybe (h ** w ** Map h w)
|
||||
parseInput inp = do
|
||||
(h ** w ** grid) <- parseGrid inp
|
||||
|
@ -21,6 +23,7 @@ parseInput inp = do
|
|||
|
||||
--- DATA
|
||||
|
||||
export
|
||||
frequencies : Map h w -> List Char
|
||||
frequencies mp = nub $ do
|
||||
row <- toList mp
|
||||
|
|
49
src/Day8/Part2.idr
Normal file
49
src/Day8/Part2.idr
Normal file
|
@ -0,0 +1,49 @@
|
|||
module Day8.Part2
|
||||
|
||||
import Data.List
|
||||
import Data.Vect
|
||||
|
||||
import Day8.Part1
|
||||
import Utils
|
||||
|
||||
%default total
|
||||
|
||||
--- DATA
|
||||
|
||||
antinodePos : {h, w : _} -> (a, b : Pos h w) -> List (Pos h w)
|
||||
antinodePos (x, y) (x', y') = do
|
||||
let dx = cast x' - cast x
|
||||
dy = cast y' - cast y
|
||||
(dx', dy') = reduce (dx, dy)
|
||||
n <- [-(cast $ max h w)..(cast $ max h w)]
|
||||
toList $
|
||||
(,) <$> integerToFin (cast x + dx' * n) h
|
||||
<*> integerToFin (cast y + dy' * n) w
|
||||
where
|
||||
reduce : (Integer, Integer) -> (Integer, Integer)
|
||||
reduce (a, b) with (cast {to=Nat} $ abs a) | (cast {to=Nat} $ abs b)
|
||||
_ | Z | _ = (a, b)
|
||||
_ | _ | Z = (a, b)
|
||||
_ | a'@(S _) | b'@(S _) =
|
||||
let g = assert_total $ gcd a' b'
|
||||
in (a `div` cast g, b `div` cast g)
|
||||
|
||||
antinodes : {h, w : _} -> Map h w -> Char -> List (Pos h w)
|
||||
antinodes mp c = do
|
||||
let poss = do
|
||||
i <- allFins h
|
||||
j <- allFins w
|
||||
guard (index (i, j) mp == Just c)
|
||||
pure (i, j)
|
||||
p1 <- poss
|
||||
p2 <- poss
|
||||
guard (p1 /= p2)
|
||||
antinodePos p1 p2
|
||||
|
||||
--- SOLUTION
|
||||
|
||||
export
|
||||
solution : String -> Maybe Nat
|
||||
solution inp = do
|
||||
(h ** w ** mp) <- parseInput inp
|
||||
pure $ length $ nub $ frequencies mp >>= antinodes mp
|
|
@ -13,7 +13,7 @@ import AllDays
|
|||
||| The latest problem that has been solved.
|
||||
-- NOTE: UPDATE AFTER EACH SOLUTION
|
||||
latest : Problem
|
||||
latest = Pr 8 Part1
|
||||
latest = Pr 8 Part2
|
||||
|
||||
|
||||
solMap : SortedMap Problem (String -> String)
|
||||
|
|
Loading…
Reference in a new issue