Custom Query (361 matches)

Filters
 
Or
 
  
 
Columns

Show under each result:


Results (55 - 57 of 361)

Ticket Resolution Summary Owner Reporter
#137 fixed Add output highlighting/insert support for Isar and sledgehammer ("Sendback") David Aspinall David Aspinall
#138 fixed Can't insert text after locking a comment David Aspinall Evgeny Makarov
Description

Dear Proof General developers,

When I issue the proof-assert-next-command-interactive (C-c C-n) command over a comment in a Coq file, the comment is joined to the locked region and the cursor is positioned at the end of the comment. After that, I cannot insert any text: whatever I type, I get a beep and a message "Region is read-only" in the minibuffer. As far as I noticed, this only happens when I type just after I have locked a comment; after I process other Coq commands, I am able to enter text.

This happens when I am using the CVS snapshot 3.7pre070704 even with no .emacs file.

By the way, when I was writing this, the link "bug tracker" on the PG home page http://proofgeneral.inf.ed.ac.uk/ was broken.

#141 worksforme Warnings missing in proof mode in Coq David Aspinall Evgeny Makarov
Description

Dear Proof General Developers,

When Coq issues a warning inside a proof, PG shows the warning in the minibuffer, but it does not show the resulting goal.

For example:

Goal True /\ True -> True.
intro H.
destruct H as [H1 H2 H3].

After the last command, the minibuffer contains "[Coq] Warning: Unused introduction pattern : H3", but the *response* buffer is empty. The same happens if I process

Require Import Setoid.
Goal False.
setoid_replace False with True.

The minibuffer contains a truncated warning "[Coq] Warning: There are several relations of the carrier 'Prop'. The relation (P", but the response buffer is again empty.

I am not sure what the correct behavior in this case should be (should PG display the warning *and* the goal?), but the goal should probably be displayed.

I am using CVS snapshot of PG updated on September 3, 2007 and Coq trunk 10056.

Thank you, Evgeny

Note: See TracQuery for help on using queries.