-
Notifications
You must be signed in to change notification settings - Fork 2
/
Copy pathEverything.agda
34 lines (28 loc) · 1.04 KB
/
Everything.agda
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
------------------------------------------------------------------------------
-- All the DTFL modules
------------------------------------------------------------------------------
-- Common options
{-# OPTIONS --double-check #-}
{-# OPTIONS --exact-split #-}
{-# OPTIONS --guardedness #-}
{-# OPTIONS --no-sized-types #-}
{-# OPTIONS --warning=all #-}
{-# OPTIONS --warning=error #-}
-- Other options
-- {-# OPTIONS --no-universe-polymorphism #-}
-- {-# OPTIONS --safe #-}
-- {-# OPTIONS --without-K #-}
module Everything where
-- Extra stuff
open import Extra.Data.List.Induction
open import Extra.Data.List.Properties
open import Extra.Data.Nat.Induction.MathematicalInduction
open import Extra.Data.Nat.Induction.Lexicographic
open import Extra.Data.Nat.Induction.WellFounded
open import Extra.Data.Nat.Properties
open import Extra.Data.Product
open import Extra.Data.Unit
open import Extra.Relation.Binary.PreorderReasoning
open import Extra.Relation.Binary.PropositionalEquality
-- Lectures
open import README