diff HoareSoundness.agda @ 63:222dd3869ab0

remove wrong ==>
author Shinji KONO <kono@ie.u-ryukyu.ac.jp>
date Sun, 22 Dec 2019 09:15:44 +0900
parents e668962ac31a
children
line wrap: on
line diff
--- a/HoareSoundness.agda	Sat Dec 21 21:12:07 2019 +0900
+++ b/HoareSoundness.agda	Sun Dec 22 09:15:44 2019 +0900
@@ -45,9 +45,6 @@
 _\/_ : Cond -> Cond -> Cond
 b1 \/ b2 = neg (neg b1 /\ neg b2)
 
-_==>_ : Cond -> Cond -> Cond
-b1 ==> b2 = neg (b1 \/ b2)
-
 when : {X  Y  Z : Set} -> (X -> Z) -> (Y -> Z) ->
        X ⊎ Y -> Z
 when f g (inj₁ x) = f x