First Git commit

This commit is contained in:
Smaug123
2019-01-04 20:45:34 +00:00
commit a435e3764e
39 changed files with 9074 additions and 0 deletions

View File

@@ -0,0 +1,8 @@
{-# OPTIONS --safe --warning=error #-}
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import LogicalFormulae
module LogicalFormulaeProofs where
transitivity : LogicalFormulae.transitivity
transitivity refl refl = refl