Minor improvement

amethyst
mueck 8 months ago
parent 1f956e528e
commit 9f77d69dcf
No known key found for this signature in database

@ -1,14 +1,12 @@
From stdpp Require Import gmap base relations. From stdpp Require Import gmap base relations.
From iris Require Import prelude. 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 *) (** * Big-step semantics *)
Implicit Types Implicit Types
(Γ : typing_context)
(v : val) (v : val)
(e : expr) (e : expr).
(A : type).
Inductive big_step : expr val Prop := Inductive big_step : expr val Prop :=
| bs_lit (n : Z) : | bs_lit (n : Z) :

Loading…
Cancel
Save