CompileCatchAll.agda 337 B

12345678910111213141516
  1. {-# OPTIONS -v treeless:20 #-}
  2. module _ where
  3. open import Common.Prelude
  4. f : List Nat → List Nat → Nat
  5. f _ [] = 0
  6. f [] (y ∷ ys) = y
  7. f (x ∷ xs) _ = x
  8. main : IO Unit
  9. main = printNat (f [] [])
  10. ,, printNat (f (1 ∷ []) [])
  11. ,, printNat (f [] (2 ∷ []))
  12. ,, printNat (f (3 ∷ []) (4 ∷ []))