Skip to content
New issue

Have a question about this project? # for a free GitHub account to open an issue and contact its maintainers and the community.

By clicking “#”, you agree to our terms of service and privacy statement. We’ll occasionally send you account related emails.

Already on GitHub? # to your account

Iris context line break incorrectly formatted #948

Closed
rongcuid opened this issue Nov 26, 2024 · 2 comments · Fixed by #984
Closed

Iris context line break incorrectly formatted #948

rongcuid opened this issue Nov 26, 2024 · 2 comments · Fixed by #984
Labels
bug Something isn't working

Comments

@rongcuid
Copy link

See also: https://gitlab.mpi-sws.org/iris/iris/-/issues/581

With Iris, the context output is incorrectly formatted.

Lemma asm (P : iProp Σ) : P ⊢ P.
Proof.
  (**
    To enter the Iris Proof Mode, we can use the tactic [iStartProof].
    However, most Iris tactics will automatically start the Iris Proof
    Mode for you, so we can directly introduce [P].
  *)
  iIntros "H".
  (**
    This adds [P] to the spatial context with the identifier ["H"]. To
    finish the proof, one would normally use either [exact] or [apply].
    So in Iris, we use either [iExact] or [iApply].
  *)
  iApply "H".
Qed.

Output:

image

The separator --- should be on its own line.

@rongcuid
Copy link
Author

rongcuid commented Dec 6, 2024

coqtop seems to be generating the correct output:

asm <   iIntros "H".
1 goal

  Σ : gFunctors
  P : iProp Σ
  ============================
  "H" : P
  --------------------------------------∗
  P

This makes Iris very hard to use

Maybe related to #852.

@gares
Copy link
Member

gares commented Dec 6, 2024

Looks loke a bug, thanks for reporting

@rtetley rtetley added the bug Something isn't working label Jan 16, 2025
# for free to join this conversation on GitHub. Already have an account? # to comment
Labels
bug Something isn't working
Projects
None yet
Development

Successfully merging a pull request may close this issue.

3 participants