|
|
|
@ -1,14 +1,12 @@
|
|
|
|
|
From stdpp Require Import gmap base relations.
|
|
|
|
|
From iris Require Import prelude.
|
|
|
|
|
From semantics.ts.stlc_extended Require Import lang notation types.
|
|
|
|
|
From semantics.ts.stlc_extended Require Import lang notation.
|
|
|
|
|
|
|
|
|
|
(** * Big-step semantics *)
|
|
|
|
|
|
|
|
|
|
Implicit Types
|
|
|
|
|
(Γ : typing_context)
|
|
|
|
|
(v : val)
|
|
|
|
|
(e : expr)
|
|
|
|
|
(A : type).
|
|
|
|
|
(e : expr).
|
|
|
|
|
|
|
|
|
|
Inductive big_step : expr → val → Prop :=
|
|
|
|
|
| bs_lit (n : Z) :
|
|
|
|
|