annotate src/axiom-taut.agda.replaced @ 1:73127e0ab57c

(none)
author soto@cr.ie.u-ryukyu.ac.jp
date Tue, 08 Sep 2020 18:38:08 +0900
parents
children
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
rev   line source
1
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
1 _@$\Rightarrow$@_ : Bool @$\rightarrow$@ Bool @$\rightarrow$@ Bool
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
2 false @$\Rightarrow$@ _ = true
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
3 true @$\Rightarrow$@ true = true
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
4 true @$\Rightarrow$@ false = false
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
5
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
6 Axiom : Cond @$\rightarrow$@ PrimComm @$\rightarrow$@ Cond @$\rightarrow$@ Set
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
7 Axiom pre comm post = @$\forall$@ (env : Env) @$\rightarrow$@ (pre env) @$\Rightarrow$@ ( post (comm env)) @$\equiv$@ true
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
8
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
9 Tautology : Cond @$\rightarrow$@ Cond @$\rightarrow$@ Set
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
10 Tautology pre post = @$\forall$@ (env : Env) @$\rightarrow$@ (pre env) @$\Rightarrow$@ (post env) @$\equiv$@ true