20 lines
313 B
Coq
20 lines
313 B
Coq
|
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 :=
|
||
|
.
|