Theory ILL
section‹Intuitionistic Linear Logic›
theory ILL
imports
Main
"HOL-Combinatorics.Permutations"
begin
text‹
Note that in this theory we often use procedural proofs rather than structured ones.
We find these to be more informative about how the basic rules of the logic are used when
compared to collecting all the rules in one call of an automated method.
›
subsection‹Deep Embedding of Propositions›
text‹
We formalise ILL propositions as a datatype, parameterised by the type of propositional variables.
The propositions are:
▪ Propositional variables
▪ Times of two terms, with unit @{text 𝟭}
▪ With of two terms, with unit @{text ⊤}
▪ Plus of two terms, with unit @{text 𝟬}
▪ Linear implication, with no unit
▪ Exponential of a term
›