Idris2/tests/idris2/reg/reg027/pwhere.idr
2023-09-07 14:57:22 +01:00

14 lines
192 B
Idris

module Main
import Data.So
total
lem1 : So x -> So (not x) -> Void
lem1 Oh Oh impossible
foo : Nat -> Int
foo z = 94
where
lem2 : So x -> So (not x) -> Void
lem2 Oh Oh impossible