mirror of
https://github.com/NixOS/nixpkgs.git
synced 2025-11-10 09:43:30 +01:00
- land `HelloWorld.agda` and `TrivialBackend.hs` in files - replace `runCommand` by `stdenvNoCC.mkDerivation` - refactor asserts
6 lines
108 B
Agda
6 lines
108 B
Agda
{-# OPTIONS --guardedness #-}
|
||
open import IO
|
||
open import Level
|
||
|
||
main = run {0ℓ} (putStrLn "Hello World!")
|