Skip to content

Instantly share code, notes, and snippets.

Show Gist options
  • Save yoshihiro503/b9bc446e0f5e0290ce442ee649a4d97c to your computer and use it in GitHub Desktop.
Save yoshihiro503/b9bc446e0f5e0290ce442ee649a4d97c to your computer and use it in GitHub Desktop.
From mathcomp Require Import all_ssreflect.
Require Import JMeq.
Inductive sizseq (T:Type) : nat -> Type :=
| SizNil : sizseq T 0
| SizCons n : T -> sizseq T n -> sizseq T n.+1.
Lemma sizseq0nil_aux (T:Type) n : forall xs : sizseq T n, n = 0 -> JMeq xs (SizNil T).
Proof.
move=> xs. now case_eq xs.
Qed.
Lemma sizseq0nil (T:Type) : all_equal_to (@SizNil T).
Proof.
move=> xs. exact/JMeq_eq/sizseq0nil_aux.
Qed.
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment