Documentation

Mathlib.Logic.Equiv.Bool

Equivalences involving Bool #

This file shows that not : BoolBool is an equivalence and derives some consequences

The boolean negation function not : BoolBool is an involution and thus an equivalence.

Equations
Instances For
    @[simp]
    theorem Equiv.boolNot_apply (a✝ : Bool) :
    boolNot a✝ = !a✝
    @[simp]
    theorem Equiv.boolNot_symm_apply (a✝ : Bool) :
    (Equiv.symm boolNot) a✝ = !a✝