Skip to content
Snippets Groups Projects
Commit fe82f3a4 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Simplify proof of fixpoint_unique.

parent 738d8bcc
No related branches found
No related tags found
No related merge requests found
...@@ -198,11 +198,9 @@ Section fixpoint. ...@@ -198,11 +198,9 @@ Section fixpoint.
Lemma fixpoint_unique (x : A) : x f x x fixpoint f. Lemma fixpoint_unique (x : A) : x f x x fixpoint f.
Proof. Proof.
rewrite !equiv_dist=> Hx n. rewrite !equiv_dist=> Hx n. induction n as [|n IH]; simpl in *.
rewrite fixpoint_eq /fixpoint_def (conv_compl n (fixpoint_chain f)) //=. - rewrite Hx fixpoint_unfold; eauto using contractive_0.
induction n as [|n IH]; simpl in *. - rewrite Hx fixpoint_unfold. apply (contractive_S _), IH.
- rewrite Hx; eauto using contractive_0.
- rewrite Hx. apply (contractive_S _), IH.
Qed. Qed.
Lemma fixpoint_ne (g : A A) `{!Contractive g} n : Lemma fixpoint_ne (g : A A) `{!Contractive g} n :
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment