Skip to content

Style for lower/upper case for initial letter in denotations #2417

Open
@mechvel

Description

@mechvel

Let Prime, Prime' : Pred ℕ _.
Then
(1) prime-2 : Prime 2
starts with the lower case letter, because is is a function.
Further,
(2) prime⇒Prime' : Prime ⇒ Prime'
has to start with a lower case letter, because it is a function.

(3) ¬Prime[0] : ¬ Prime 0
starts with a lower case letter, because it is a function,
and the second letter is preserved in the upper case, because it is of the type name.

These are my suggestions for the style.
In some places in lib-2.1-rc1 the rules (2) and (3) are satisfied, and in some other places they are broken.

I suggest the rules (1), (2), (3),
have a large code that follows these rules, while lib-2* looks neutral relatively to (2), (3).
Can the team take this style for future?

Metadata

Metadata

Assignees

No one assigned

    Labels

    Type

    No type

    Projects

    No projects

    Milestone

    No milestone

    Relationships

    None yet

    Development

    No branches or pull requests

    Issue actions