File: Main.agda

package info (click to toggle)
agda-stdlib 2.1-4
  • links: PTS, VCS
  • area: main
  • in suites: forky, sid, trixie
  • size: 9,196 kB
  • sloc: haskell: 375; makefile: 32; sh: 28; lisp: 1
file content (39 lines) | stat: -rw-r--r-- 848 bytes parent folder | download
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
{-# OPTIONS --guardedness --sized-types #-}

module Main where

open import Data.List.Base using (_∷_; [])
open import Data.String.Base using (String; unlines)
open import Data.Tree.Rose
open import Data.Tree.Rose.Show
open import IO.Base
open import IO.Finite
open import Function.Base using (_$_; id)

dependencies : Rose String _
dependencies = node "standard-library"
  $ agda
  ∷ cabal
  ∷ haskell
  ∷ [] where

  haskell : Rose String _
  haskell = node "Haskell"
    $ node "Haskell (bootstrap)" []
    ∷ node "C" []
    ∷ []

  cabal : Rose String _
  cabal = node "cabal" (haskell ∷ [])

  agda : Rose String _
  agda = node "Agda"
    $ haskell
    ∷ cabal
    ∷ node "alex" (haskell ∷ [])
    ∷ node "happy" (haskell ∷ [])
    ∷ []

main : Main
main = run $ do
  putStrLn $ unlines $ showSimple id dependencies