Files
agdaproofs/Logic/PropositionalAxiomsTautology.agda
2019-02-19 08:31:46 +00:00

12 lines
287 B
Agda

{-# OPTIONS --safe --warning=error #-}
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import LogicalFormulae
open import Logic.PropositionalLogic
open import Functions
open import Numbers.Naturals
open import Vectors
module Logic.PropositionalAxiomsTautology where