From ae0b57980df2dbdc8bc5a6f6049ead724964d441 Mon Sep 17 00:00:00 2001 From: Robbert Krebbers <mail@robbertkrebbers.nl> Date: Thu, 2 Apr 2020 11:01:16 +0200 Subject: [PATCH] Break some very long lines in `class_instances_bi`. --- theories/proofmode/class_instances_bi.v | 7 +++++-- 1 file changed, 5 insertions(+), 2 deletions(-) diff --git a/theories/proofmode/class_instances_bi.v b/theories/proofmode/class_instances_bi.v index f4c47e62c..3edfef488 100644 --- a/theories/proofmode/class_instances_bi.v +++ b/theories/proofmode/class_instances_bi.v @@ -698,7 +698,8 @@ Qed. Global Instance into_and_sep `{BiPositive PROP} P Q : IntoAnd true (P ∗ Q) P Q. Proof. - rewrite /IntoAnd /= intuitionistically_sep -and_sep_intuitionistically intuitionistically_and //. + rewrite /IntoAnd /= intuitionistically_sep + -and_sep_intuitionistically intuitionistically_and //. Qed. Global Instance into_and_sep_affine P Q : TCOr (Affine P) (Absorbing Q) → TCOr (Absorbing P) (Affine Q) → @@ -990,7 +991,9 @@ Global Instance into_forall_wand P Q : Proof. rewrite /IntoForall. apply forall_intro=><-. rewrite emp_wand //. Qed. Global Instance into_forall_impl `{!BiAffine PROP} P Q : IntoForall (P → Q) (λ _ : ⊢ P, Q) | 10. -Proof. rewrite /IntoForall. apply forall_intro=><-. rewrite -True_emp True_impl //. Qed. +Proof. + rewrite /IntoForall. apply forall_intro=><-. rewrite -True_emp True_impl //. +Qed. (** FromForall *) Global Instance from_forall_forall {A} (Φ : A → PROP) : -- GitLab