Minor
This commit is contained in:
parent
eaf59fc45e
commit
8daaae9831
1 changed files with 24 additions and 1 deletions
|
@ -998,7 +998,7 @@ Proof.
|
||||||
apply : bind_inst; eauto.
|
apply : bind_inst; eauto.
|
||||||
Qed.
|
Qed.
|
||||||
|
|
||||||
Lemma coqeq_complete n k (a b : PTm n) :
|
Lemma coqeq_complete' n k (a b : PTm n) :
|
||||||
algo_metric k a b ->
|
algo_metric k a b ->
|
||||||
(forall Γ A, Γ ⊢ a ∈ A -> Γ ⊢ b ∈ A -> a ⇔ b) /\
|
(forall Γ A, Γ ⊢ a ∈ A -> Γ ⊢ b ∈ A -> a ⇔ b) /\
|
||||||
(forall Γ A B, ishne a -> ishne b -> Γ ⊢ a ∈ A -> Γ ⊢ b ∈ B -> a ∼ b /\ exists C, Γ ⊢ C ≲ A /\ Γ ⊢ C ≲ B /\ Γ ⊢ a ∈ C /\ Γ ⊢ b ∈ C).
|
(forall Γ A B, ishne a -> ishne b -> Γ ⊢ a ∈ A -> Γ ⊢ b ∈ B -> a ∼ b /\ exists C, Γ ⊢ C ≲ A /\ Γ ⊢ C ≲ B /\ Γ ⊢ a ∈ C /\ Γ ⊢ b ∈ C).
|
||||||
|
@ -1323,3 +1323,26 @@ Proof.
|
||||||
* sfirstorder use:T_Bot_Imp.
|
* sfirstorder use:T_Bot_Imp.
|
||||||
+ sfirstorder use:T_Bot_Imp.
|
+ sfirstorder use:T_Bot_Imp.
|
||||||
Qed.
|
Qed.
|
||||||
|
|
||||||
|
Lemma coqeq_sound : forall n Γ (a b : PTm n) A,
|
||||||
|
Γ ⊢ a ∈ A -> Γ ⊢ b ∈ A -> a ⇔ b -> Γ ⊢ a ≡ b ∈ A.
|
||||||
|
Proof. sfirstorder use:coqeq_sound_mutual. Qed.
|
||||||
|
|
||||||
|
Lemma coqeq_complete n Γ (a b A : PTm n) :
|
||||||
|
Γ ⊢ a ≡ b ∈ A -> a ⇔ b.
|
||||||
|
Proof.
|
||||||
|
move => h.
|
||||||
|
suff : exists k, algo_metric k a b by hauto lq:on use:coqeq_complete', regularity.
|
||||||
|
eapply fundamental_theorem in h.
|
||||||
|
move /logrel.SemEq_SN_Join : h.
|
||||||
|
move => h.
|
||||||
|
have : exists va vb : PTm n,
|
||||||
|
rtc LoRed.R a va /\
|
||||||
|
rtc LoRed.R b vb /\ nf va /\ nf vb /\ EJoin.R va vb
|
||||||
|
by hauto l:on use:DJoin.standardization_lo.
|
||||||
|
move => [va][vb][hva][hvb][nva][nvb]hj.
|
||||||
|
move /relations.rtc_nsteps : hva => [i hva].
|
||||||
|
move /relations.rtc_nsteps : hvb => [j hvb].
|
||||||
|
exists (i + j + size_PTm va + size_PTm vb).
|
||||||
|
hauto lq:on solve+:lia.
|
||||||
|
Qed.
|
||||||
|
|
Loading…
Add table
Add a link
Reference in a new issue