From Undecidability.TM Require Import TM Util.TM_facts HoareLogic HoareRegister.

Lemma RealiseIntroAll sig F n X (P : _ _ _ _, Prop) (M : pTM sig F n):
  ( x, M ( tin '(yout, tout) P x tin yout tout))
  M ( tin '(yout, tout) (x:X), P x tin yout tout).
Proof.
  unfold Realise. intros. firstorder.
Qed.


Lemma TerminatesInIntroEx sig n X (T : _ _ _, Prop) (M : TM sig n):
  ( x, M ( tin k T x tin k))
  M ( tin k (x:X), T x tin k).
Proof.
  unfold TerminatesIn. intros. firstorder.
Qed.