Skip to content
Snippets Groups Projects
Commit 3c495d6d authored by Jacques-Henri Jourdan's avatar Jacques-Henri Jourdan
Browse files

Tweak.

parent f3cce8a0
No related branches found
No related tags found
No related merge requests found
Pipeline #
......@@ -56,8 +56,8 @@ Section fn.
pointwise_relation A (dist n') ==> dist n') (fn E).
Proof.
intros ?? H1 ?? H2.
apply fn_contractive=>u; destruct n'; try done; apply dist_S.
by apply (H1 u). by apply (H2 u).
apply fn_contractive=>u; (destruct n'; [done|apply dist_S]);
[apply (H1 u)|apply (H2 u)].
Qed.
End fn.
......
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