oplss2024/zdancewic/Day1.v

20 lines
313 B
Coq
Raw Normal View History

2024-06-11 02:56:36 +00:00
Require Import Coq.Strings.String.
Module Day1.
Inductive aexp : Type :=
.
Inductive bexp : Type :=
.
Inductive com : Type :=
| CSkip
| CAssign (x : string) (a : aexp)
| CSeq (c1 c2 : com)
| CIf (b : bexp) (c1 c2 : com)
| CWhile (b : bexp) (c : com)
.
Fixpoint aeval (m : mem) (a : aexp) : nat :=
.