Files
agdaproofs/Everything/Unsafe.agda
2019-12-07 13:00:18 +00:00

8 lines
189 B
Agda

{-# OPTIONS --warning=error --allow-unsolved-metas #-}
-- This file contains everything that cannot be compiled in --safe mode.
open import Lists.SortList
module Everything.Unsafe where