RELAX-NG Schema Documentation


Table of Contents

Grammar Documentation
Element: Abstractness
Element: Adjective
Element: And
Element: Antisymmetry
Element: ArgTypes
Element: Article
Element: ArticleID
Element: Associativity
Element: Assume
Element: BlockThesis
Element: By
Element: CCluster
Element: Canceled
Element: Case
Element: CaseBlock
Element: Cluster
Element: Coherence
Element: Commutativity
Element: Compatibility
Element: Conclusion
Element: Connectedness
Element: Consider
Element: Consistency
Element: Const
Element: ConstrCount
Element: ConstrCounts
Element: Constructor
Element: Constructors
Element: Correctness
Element: DefFunc
Element: DefMeaning
Element: DefPred
Element: DefTheorem
Element: Definiens
Element: Definientia
Element: Definition
Element: DefinitionBlock
Element: EndPosition
Element: ErrorCluster
Element: ErrorFrm
Element: ErrorInf
Element: ErrorTrm
Element: Essentials
Element: Existence
Element: Expansion
Element: FCluster
Element: Fields
Element: For
Element: Format
Element: Formats
Element: Fraenkel
Element: FreeVar
Element: From
Element: Func
Element: Given
Element: Idempotence
Element: InfConst
Element: Int
Element: Involutiveness
Element: Irreflexivity
Element: Is
Element: It
Element: IterEquality
Element: IterStep
Element: JustifiedProperty
Element: JustifiedTheorem
Element: LambdaVar
Element: Let
Element: LocusVar
Element: Not
Element: NotationBlock
Element: Notations
Element: Now
Element: Num
Element: Pair
Element: PartialDef
Element: Pattern
Element: PerCases
Element: PerCasesReasoning
Element: Pred
Element: Priority
Element: PrivFunc
Element: PrivPred
Element: Projectivity
Element: Proof
Element: Properties
Element: Proposition
Element: QuaTrm
Element: RCluster
Element: Reconsider
Element: Ref
Element: Reflexivity
Element: Registration
Element: RegistrationBlock
Element: Registrations
Element: Requirement
Element: Requirements
Element: Reservation
Element: Scheme
Element: SchemeBlock
Element: SchemeFuncDecl
Element: SchemePredDecl
Element: SchemePremises
Element: Schemes
Element: Set
Element: Signature
Element: SignatureWithCounts
Element: SkippedProof
Element: StructLoci
Element: Suppose
Element: SupposeBlock
Element: Symbol
Element: SymbolCount
Element: Symbols
Element: Symmetry
Element: Take
Element: TakeAsVar
Element: Theorem
Element: Theorems
Element: Thesis
Element: ThesisExpansions
Element: Transitivity
Element: Typ
Element: UnexpectedProp
Element: Uniqueness
Element: UnknownCorrCond
Element: Var
Element: Verum
Element: Visible
Element: Vocabularies
Element: Vocabulary
Pattern: Adjective
Pattern: And
Pattern: ArgTypes
Pattern: Article
Pattern: ArticleID
Pattern: Assume
Pattern: AuxiliaryItem
Pattern: BlockThesis
Pattern: By
Pattern: CCluster
Pattern: Canceled
Pattern: Case
Pattern: CaseBlock
Pattern: Cluster
Pattern: Coherence
Pattern: Compatibility
Pattern: Conclusion
Pattern: Consider
Pattern: Consistency
Pattern: Const
Pattern: ConstrCounts
Pattern: Constructor
Pattern: Constructors
Pattern: Correctness
Pattern: CorrectnessCondition
Pattern: DefFunc
Pattern: DefMeaning
Pattern: DefPred
Pattern: DefTheorem
Pattern: Definiens
Pattern: Definientia
Pattern: Definition
Pattern: DefinitionBlock
Pattern: EndPosition
Pattern: ErrorCluster
Pattern: ErrorFrm
Pattern: ErrorTrm
Pattern: Existence
Pattern: FCluster
Pattern: Fields
Pattern: For
Pattern: Format
Pattern: Formats
Pattern: Formula
Pattern: Fraenkel
Pattern: FreeVar
Pattern: From
Pattern: Func
Pattern: Given
Pattern: InfConst
Pattern: Inference
Pattern: Int
Pattern: Is
Pattern: It
Pattern: IterEquality
Pattern: IterStep
Pattern: Justification
Pattern: JustifiedProperty
Pattern: JustifiedProposition
Pattern: JustifiedTheorem
Pattern: LambdaVar
Pattern: Let
Pattern: LocusVar
Pattern: Not
Pattern: NotationBlock
Pattern: Notations
Pattern: Now
Pattern: Num
Pattern: Pair
Pattern: Pattern
Pattern: PerCases
Pattern: PerCasesReasoning
Pattern: Position
Pattern: Pred
Pattern: PrivFunc
Pattern: PrivPred
Pattern: Proof
Pattern: Properties
Pattern: Property
Pattern: Proposition
Pattern: QuaTrm
Pattern: RCluster
Pattern: Reasoning
Pattern: Reconsider
Pattern: Ref
Pattern: Registration
Pattern: RegistrationBlock
Pattern: Registrations
Pattern: Requirements
Pattern: Reservation
Pattern: Scheme
Pattern: SchemeBlock
Pattern: SchemeFuncDecl
Pattern: SchemePredDecl
Pattern: Schemes
Pattern: Set
Pattern: Signature
Pattern: SkeletonItem
Pattern: SkippedProof
Pattern: StructLoci
Pattern: Suppose
Pattern: SupposeBlock
Pattern: Symbols
Pattern: Take
Pattern: TakeAsVar
Pattern: Term
Pattern: Theorems
Pattern: Thesis
Pattern: ThesisExpansions
Pattern: Typ
Pattern: Uniqueness
Pattern: UnknownCorrCond
Pattern: Var
Pattern: Verum
Pattern: Vocabularies

Grammar Documentation

Namespace:

Element: Abstractness

Table 1. Element: Abstractness

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Abstractness" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Adjective

Table 2. Element: Adjective

Documentation

No documentation available.

Content Model

( %Term; )*

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

value xsd:booleanOptional

Source

<element name="Adjective" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <optional>
        <attribute name="value">
          <data type="boolean"/>
        </attribute>
      </optional>
      <zeroOrMore>
        <ref name="Term"/>
      </zeroOrMore>
    </element>

Element: And

Table 3. Element: And

Documentation

No documentation available.

Content Model

( %Formula; )*

Source

<element name="And" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="Formula"/>
      </zeroOrMore>
    </element>

Element: Antisymmetry

Table 4. Element: Antisymmetry

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Antisymmetry" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: ArgTypes

Table 5. Element: ArgTypes

Documentation

No documentation available.

Content Model

( %Typ; )*

Source

<element name="ArgTypes" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="Typ"/>
      </zeroOrMore>
    </element>

Element: Article

Table 6. Element: Article

Documentation

No documentation available.

Content Model

( ( %DefinitionBlock; | %RegistrationBlock; | %NotationBlock; | %Reservation; | %SchemeBlock; | %JustifiedTheorem; | %DefTheorem; | %Definiens; | %Canceled; | %Pattern; | %AuxiliaryItem; ) )*

Attributes

Attribute

Type

Use

Documentation

aid xsd:stringOptional

Source

<element name="Article" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="aid">
        <data type="string"/>
      </attribute>
      <zeroOrMore>
        <choice>
          <ref name="DefinitionBlock"/>
          <ref name="RegistrationBlock"/>
          <ref name="NotationBlock"/>
          <ref name="Reservation"/>
          <ref name="SchemeBlock"/>
          <ref name="JustifiedTheorem"/>
          <ref name="DefTheorem"/>
          <ref name="Definiens"/>
          <ref name="Canceled"/>
          <ref name="Pattern"/>
          <ref name="AuxiliaryItem"/>
        </choice>
      </zeroOrMore>
    </element>

Element: ArticleID

Table 7. Element: ArticleID

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

name xsd:stringOptional

Source

<element name="ArticleID" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="name">
        <data type="string"/>
      </attribute>
    </element>

Element: Associativity

Table 8. Element: Associativity

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Associativity" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Assume

Table 9. Element: Assume

Documentation

No documentation available.

Content Model

( %Proposition; )+

Source

<element name="Assume" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <oneOrMore>
        <ref name="Proposition"/>
      </oneOrMore>
    </element>

Element: BlockThesis

Table 10. Element: BlockThesis

Documentation

No documentation available.

Content Model

%Formula;

Source

<element name="BlockThesis" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Formula"/>
    </element>

Element: By

Table 11. Element: By

Documentation

No documentation available.

Content Model

( %Ref; )*

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

linked xsd:booleanOptional

Source

<element name="By" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <optional>
        <attribute name="linked">
          <data type="boolean"/>
        </attribute>
      </optional>
      <zeroOrMore>
        <ref name="Ref"/>
      </zeroOrMore>
    </element>

Element: CCluster

Table 12. Element: CCluster

Documentation

No documentation available.

Content Model

( %ErrorCluster; | ( %ArgTypes; %Cluster; %Typ; %Cluster; ) )

Source

<element name="CCluster" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="ErrorCluster"/>
        <group>
          <ref name="ArgTypes"/>
          <ref name="Cluster"/>
          <ref name="Typ"/>
          <ref name="Cluster"/>
        </group>
      </choice>
    </element>

Element: Canceled

Table 13. Element: Canceled

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Canceled" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <empty/>
    </element>

Element: Case

Table 14. Element: Case

Documentation

No documentation available.

Content Model

( %Proposition; )+

Source

<element name="Case" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <oneOrMore>
        <ref name="Proposition"/>
      </oneOrMore>
    </element>

Element: CaseBlock

Table 15. Element: CaseBlock

Documentation

No documentation available.

Content Model

( ( %BlockThesis; %Case; %Thesis; %Reasoning; ) | ( %Case; %Reasoning; %BlockThesis; ) )

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="CaseBlock" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <choice>
        <group>
          <ref name="BlockThesis"/>
          <ref name="Case"/>
          <ref name="Thesis"/>
          <ref name="Reasoning"/>
        </group>
        <group>
          <ref name="Case"/>
          <ref name="Reasoning"/>
          <ref name="BlockThesis"/>
        </group>
      </choice>
    </element>

Element: Cluster

Table 16. Element: Cluster

Documentation

No documentation available.

Content Model

( %Adjective; )*

Source

<element name="Cluster" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="Adjective"/>
      </zeroOrMore>
    </element>

Element: Coherence

Table 17. Element: Coherence

Documentation

No documentation available.

Content Model

( %Formula; | ( %Proposition; %Justification; ) )

Source

<element name="Coherence" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="Formula"/>
        <group>
          <ref name="Proposition"/>
          <ref name="Justification"/>
        </group>
      </choice>
    </element>

Element: Commutativity

Table 18. Element: Commutativity

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Commutativity" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Compatibility

Table 19. Element: Compatibility

Documentation

No documentation available.

Content Model

( %Formula; | ( %Proposition; %Justification; ) )

Source

<element name="Compatibility" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="Formula"/>
        <group>
          <ref name="Proposition"/>
          <ref name="Justification"/>
        </group>
      </choice>
    </element>

Element: Conclusion

Table 20. Element: Conclusion

Documentation

No documentation available.

Content Model

%JustifiedProposition;

Source

<element name="Conclusion" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="JustifiedProposition"/>
    </element>

Element: Connectedness

Table 21. Element: Connectedness

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Connectedness" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Consider

Table 22. Element: Consider

Documentation

No documentation available.

Content Model

%Proposition;, %Justification;, ( %Typ; )+ , ( %Proposition; )*

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="Consider" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <ref name="Proposition"/>
      <ref name="Justification"/>
      <oneOrMore>
        <ref name="Typ"/>
      </oneOrMore>
      <zeroOrMore>
        <ref name="Proposition"/>
      </zeroOrMore>
    </element>

Element: Consistency

Table 23. Element: Consistency

Documentation

No documentation available.

Content Model

( %Formula; | ( %Proposition; %Justification; ) )

Source

<element name="Consistency" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="Formula"/>
        <group>
          <ref name="Proposition"/>
          <ref name="Justification"/>
        </group>
      </choice>
    </element>

Element: Const

Table 24. Element: Const

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="Const" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
    </element>

Element: ConstrCount

Table 25. Element: ConstrCount

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "M" | "L" | "V" | "R" | "K" | "U" | "G" Optional

nr xsd:integerOptional

Source

<element name="ConstrCount" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
          <attribute name="kind">
            <choice>
              <value>M</value>
              <value>L</value>
              <value>V</value>
              <value>R</value>
              <value>K</value>
              <value>U</value>
              <value>G</value>
            </choice>
          </attribute>
          <attribute name="nr">
            <data type="integer"/>
          </attribute>
        </element>

Element: ConstrCounts

Table 26. Element: ConstrCounts

Documentation

No documentation available.

Content Model

( ConstrCount )*

Attributes

Attribute

Type

Use

Documentation

name xsd:stringOptional

Source

<element name="ConstrCounts" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="name">
          <data type="string"/>
        </attribute>
      </optional>
      <zeroOrMore>
        <element name="ConstrCount">
          <attribute name="kind">
            <choice>
              <value>M</value>
              <value>L</value>
              <value>V</value>
              <value>R</value>
              <value>K</value>
              <value>U</value>
              <value>G</value>
            </choice>
          </attribute>
          <attribute name="nr">
            <data type="integer"/>
          </attribute>
        </element>
      </zeroOrMore>
    </element>

Element: Constructor

Table 27. Element: Constructor

Documentation

No documentation available.

Content Model

%Properties; ? , %ArgTypes;, %StructLoci; ? , ( %Typ; )* , %Fields; ?

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "M" | "L" | "V" | "R" | "K" | "U" | "G" Optional

nr xsd:integerOptional

aid xsd:stringOptional

relnr xsd:integerOptional

redefnr xsd:integerOptional

superfluous xsd:integerOptional

structmodeaggrnr xsd:integerOptional

aggregbase xsd:integerOptional

Source

<element name="Constructor" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="kind">
        <choice>
          <value>M</value>
          <value>L</value>
          <value>V</value>
          <value>R</value>
          <value>K</value>
          <value>U</value>
          <value>G</value>
        </choice>
      </attribute>
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <attribute name="aid">
        <data type="string"/>
      </attribute>
      <optional>
        <attribute name="relnr">
          <data type="integer"/>
        </attribute>
      </optional>
      <optional>
        <attribute name="redefnr">
          <data type="integer"/>
        </attribute>
        <attribute name="superfluous">
          <data type="integer"/>
        </attribute>
      </optional>
      <optional>
        <choice>
          <attribute name="structmodeaggrnr">
            <data type="integer"/>
          </attribute>
          <attribute name="aggregbase">
            <data type="integer"/>
          </attribute>
        </choice>
      </optional>
      <optional>
        <ref name="Properties"/>
      </optional>
      <ref name="ArgTypes"/>
      <optional>
        <ref name="StructLoci"/>
      </optional>
      <zeroOrMore>
        <ref name="Typ"/>
      </zeroOrMore>
      <optional>
        <ref name="Fields"/>
      </optional>
    </element>

Element: Constructors

Table 28. Element: Constructors

Documentation

No documentation available.

Content Model

( SignatureWithCounts | ( %Signature; %ConstrCounts; ) ) ? , ( %Constructor; )*

Attributes

Attribute

Type

Use

Documentation

aid xsd:stringOptional

Source

<element name="Constructors" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="aid">
          <data type="string"/>
        </attribute>
      </optional>
      <optional>
        <choice>
          <element name="SignatureWithCounts">
            <zeroOrMore>
              <ref name="ConstrCounts"/>
            </zeroOrMore>
          </element>
          <group>
            <ref name="Signature"/>
            <ref name="ConstrCounts"/>
          </group>
        </choice>
      </optional>
      <zeroOrMore>
        <ref name="Constructor"/>
      </zeroOrMore>
    </element>

Element: Correctness

Table 29. Element: Correctness

Documentation

No documentation available.

Content Model

( %CorrectnessCondition; )* %Proposition; %Justification;

Source

<element name="Correctness" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="CorrectnessCondition"/>
      </zeroOrMore>
      <ref name="Proposition"/>
      <ref name="Justification"/>
    </element>

Element: DefFunc

Table 30. Element: DefFunc

Documentation

No documentation available.

Content Model

%ArgTypes; %Term; %Typ;

Source

<element name="DefFunc" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="ArgTypes"/>
      <ref name="Term"/>
      <ref name="Typ"/>
    </element>

Element: DefMeaning

Table 31. Element: DefMeaning

Documentation

No documentation available.

Content Model

( PartialDef )* , ( %Formula; | %Term; ) ?

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "e" | "m" Optional

Source

<element name="DefMeaning" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="kind">
        <choice>
          <value>e</value>
          <value>m</value>
        </choice>
      </attribute>
      <zeroOrMore>
        <element name="PartialDef">
          <choice>
            <ref name="Formula"/>
            <ref name="Term"/>
          </choice>
          <ref name="Formula"/>
        </element>
      </zeroOrMore>
      <optional>
        <choice>
          <ref name="Formula"/>
          <ref name="Term"/>
        </choice>
      </optional>
    </element>

Element: DefPred

Table 32. Element: DefPred

Documentation

No documentation available.

Content Model

%ArgTypes; %Formula;

Source

<element name="DefPred" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="ArgTypes"/>
      <ref name="Formula"/>
    </element>

Element: DefTheorem

Table 33. Element: DefTheorem

Documentation

No documentation available.

Content Model

%Proposition;

Source

<element name="DefTheorem" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Proposition"/>
    </element>

Element: Definiens

Table 34. Element: Definiens

Documentation

No documentation available.

Content Model

( %Typ; )* , Essentials, %Formula; ? %DefMeaning;

Attributes

Attribute

Type

Use

Documentation

constrkind Enumeration: "M" | "L" | "V" | "R" | "K" | "U" | "G" Optional

constrnr xsd:integerOptional

Source

<element name="Definiens" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="constrkind">
        <choice>
          <value>M</value>
          <value>L</value>
          <value>V</value>
          <value>R</value>
          <value>K</value>
          <value>U</value>
          <value>G</value>
        </choice>
      </attribute>
      <attribute name="constrnr">
        <data type="integer"/>
      </attribute>
      <zeroOrMore>
        <ref name="Typ"/>
      </zeroOrMore>
      <element name="Essentials">
        <zeroOrMore>
          <ref name="Int"/>
        </zeroOrMore>
      </element>
      <optional>
        <ref name="Formula"/>
      </optional>
      <ref name="DefMeaning"/>
    </element>

Element: Definientia

Table 35. Element: Definientia

Documentation

No documentation available.

Content Model

%Signature; ? , ( %Definiens; )*

Attributes

Attribute

Type

Use

Documentation

aid xsd:stringOptional

Source

<element name="Definientia" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="aid">
          <data type="string"/>
        </attribute>
      </optional>
      <optional>
        <ref name="Signature"/>
      </optional>
      <zeroOrMore>
        <ref name="Definiens"/>
      </zeroOrMore>
    </element>

Element: Definition

Table 36. Element: Definition

Documentation

No documentation available.

Content Model

? ( ( ( %CorrectnessCondition; )* , %Correctness; ? , ( %JustifiedProperty; )* , %Constructor; ? ) | ( %Constructor;, %Constructor;, ( %Constructor; )+ , ( %CorrectnessCondition; )* , %Correctness; ? ) )

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "M" | "V" | "R" | "K" | "G" Optional

redefinition xsd:booleanOptional

expandable xsd:booleanOptional

nr xsd:integerOptional

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="Definition" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="kind">
        <choice>
          <value>M</value>
          <value>V</value>
          <value>R</value>
          <value>K</value>
          <value>G</value>
        </choice>
      </attribute>
      <optional>
        <attribute name="redefinition">
          <data type="boolean"/>
        </attribute>
      </optional>
      <optional>
        <attribute name="expandable">
          <data type="boolean"/>
        </attribute>
      </optional>
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
        <ref name="Position"/>
      </optional>
      <choice>
        <group>
          <zeroOrMore>
            <ref name="CorrectnessCondition"/>
          </zeroOrMore>
          <optional>
            <ref name="Correctness"/>
          </optional>
          <zeroOrMore>
            <ref name="JustifiedProperty"/>
          </zeroOrMore>
          <optional>
            <ref name="Constructor"/>
          </optional>
        </group>
        <group>
          <ref name="Constructor"/>
          <ref name="Constructor"/>
          <oneOrMore>
            <ref name="Constructor"/>
          </oneOrMore>
          <zeroOrMore>
            <ref name="CorrectnessCondition"/>
          </zeroOrMore>
          <optional>
            <ref name="Correctness"/>
          </optional>
        </group>
      </choice>
    </element>

Element: DefinitionBlock

Table 37. Element: DefinitionBlock

Documentation

No documentation available.

Content Model

( ( %Let; | %Assume; | %Given; | %AuxiliaryItem; | %Canceled; | %Definition; ) )* %EndPosition;

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="DefinitionBlock" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <zeroOrMore>
        <choice>
          <ref name="Let"/>
          <ref name="Assume"/>
          <ref name="Given"/>
          <ref name="AuxiliaryItem"/>
          <ref name="Canceled"/>
          <ref name="Definition"/>
        </choice>
      </zeroOrMore>
      <ref name="EndPosition"/>
    </element>

Element: EndPosition

Table 38. Element: EndPosition

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="EndPosition" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
    </element>

Element: ErrorCluster

Table 39. Element: ErrorCluster

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="ErrorCluster" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <empty/>
    </element>

Element: ErrorFrm

Table 40. Element: ErrorFrm

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="ErrorFrm" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <empty/>
    </element>

Element: ErrorInf

Table 41. Element: ErrorInf

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="ErrorInf" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: ErrorTrm

Table 42. Element: ErrorTrm

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="ErrorTrm" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <empty/>
    </element>

Element: Essentials

Table 43. Element: Essentials

Documentation

No documentation available.

Content Model

( %Int; )*

Source

<element name="Essentials" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <zeroOrMore>
          <ref name="Int"/>
        </zeroOrMore>
      </element>

Element: Existence

Table 44. Element: Existence

Documentation

No documentation available.

Content Model

( %Formula; | ( %Proposition; %Justification; ) )

Source

<element name="Existence" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="Formula"/>
        <group>
          <ref name="Proposition"/>
          <ref name="Justification"/>
        </group>
      </choice>
    </element>

Element: Expansion

Table 45. Element: Expansion

Documentation

No documentation available.

Content Model

%Typ;

Source

<element name="Expansion" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
          <ref name="Typ"/>
        </element>

Element: FCluster

Table 46. Element: FCluster

Documentation

No documentation available.

Content Model

( %ErrorCluster; | ( %ArgTypes; %Term; %Cluster; ) )

Source

<element name="FCluster" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="ErrorCluster"/>
        <group>
          <ref name="ArgTypes"/>
          <ref name="Term"/>
          <ref name="Cluster"/>
        </group>
      </choice>
    </element>

Element: Fields

Table 47. Element: Fields

Documentation

No documentation available.

Content Model

( %Int; )*

Source

<element name="Fields" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="Int"/>
      </zeroOrMore>
    </element>

Element: For

Table 48. Element: For

Documentation

No documentation available.

Content Model

%Typ; %Formula;

Source

<element name="For" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Typ"/>
      <ref name="Formula"/>
    </element>

Element: Format

Table 49. Element: Format

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "G" | "K" | "J" | "L" | "M" | "O" | "R" | "U" | "V" Optional

nr xsd:integerOptional

symbolnr xsd:integerOptional

argnr xsd:integerOptional

leftargnr xsd:integerOptional

rightsymbolnr xsd:integerOptional

Source

<element name="Format" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="kind">
        <choice>
          <value>G</value>
          <value>K</value>
          <value>J</value>
          <value>L</value>
          <value>M</value>
          <value>O</value>
          <value>R</value>
          <value>U</value>
          <value>V</value>
        </choice>
      </attribute>
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <attribute name="symbolnr">
        <data type="integer"/>
      </attribute>
      <attribute name="argnr">
        <data type="integer"/>
      </attribute>
      <optional>
        <attribute name="leftargnr">
          <data type="integer"/>
        </attribute>
      </optional>
      <optional>
        <attribute name="rightsymbolnr">
          <data type="integer"/>
        </attribute>
      </optional>
    </element>

Element: Formats

Table 50. Element: Formats

Documentation

No documentation available.

Content Model

( %Format; )* , ( Priority )*

Source

<element name="Formats" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="Format"/>
      </zeroOrMore>
      <zeroOrMore>
        <element name="Priority">
          <attribute name="kind">
            <choice>
              <value>O</value>
              <value>K</value>
              <value>L</value>
            </choice>
          </attribute>
          <attribute name="symbolnr">
            <data type="integer"/>
          </attribute>
          <attribute name="value">
            <data type="integer"/>
          </attribute>
        </element>
      </zeroOrMore>
    </element>

Element: Fraenkel

Table 51. Element: Fraenkel

Documentation

No documentation available.

Content Model

( %Typ; )* %Term; %Formula;

Source

<element name="Fraenkel" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="Typ"/>
      </zeroOrMore>
      <ref name="Term"/>
      <ref name="Formula"/>
    </element>

Element: FreeVar

Table 52. Element: FreeVar

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="FreeVar" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
    </element>

Element: From

Table 53. Element: From

Documentation

No documentation available.

Content Model

( %Ref; )*

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

articlenr xsd:integerOptional

nr xsd:integerOptional

Source

<element name="From" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <attribute name="articlenr">
        <data type="integer"/>
      </attribute>
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <zeroOrMore>
        <ref name="Ref"/>
      </zeroOrMore>
    </element>

Element: Func

Table 54. Element: Func

Documentation

No documentation available.

Content Model

( %Term; )*

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "F" | "G" | "K" | "U" Optional

nr xsd:integerOptional

Source

<element name="Func" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="kind">
        <choice>
          <value>F</value>
          <value>G</value>
          <value>K</value>
          <value>U</value>
        </choice>
      </attribute>
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <zeroOrMore>
        <ref name="Term"/>
      </zeroOrMore>
    </element>

Element: Given

Table 55. Element: Given

Documentation

No documentation available.

Content Model

( %Typ; )+ , ( %Proposition; )+

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="Given" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <oneOrMore>
        <ref name="Typ"/>
      </oneOrMore>
      <oneOrMore>
        <ref name="Proposition"/>
      </oneOrMore>
    </element>

Element: Idempotence

Table 56. Element: Idempotence

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Idempotence" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: InfConst

Table 57. Element: InfConst

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="InfConst" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
    </element>

Element: Int

Table 58. Element: Int

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

x xsd:integerOptional

Source

<element name="Int" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="x">
        <data type="integer"/>
      </attribute>
    </element>

Element: Involutiveness

Table 59. Element: Involutiveness

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Involutiveness" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Irreflexivity

Table 60. Element: Irreflexivity

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Irreflexivity" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Is

Table 61. Element: Is

Documentation

No documentation available.

Content Model

%Term; %Typ;

Source

<element name="Is" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Term"/>
      <ref name="Typ"/>
    </element>

Element: It

Table 62. Element: It

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="It" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <empty/>
    </element>

Element: IterEquality

Table 63. Element: IterEquality

Documentation

No documentation available.

Content Model

%Term;, ( %IterStep; )+

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="IterEquality" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <ref name="Position"/>
      <ref name="Term"/>
      <oneOrMore>
        <ref name="IterStep"/>
      </oneOrMore>
    </element>

Element: IterStep

Table 64. Element: IterStep

Documentation

No documentation available.

Content Model

%Term; %Inference;

Source

<element name="IterStep" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Term"/>
      <ref name="Inference"/>
    </element>

Element: JustifiedProperty

Table 65. Element: JustifiedProperty

Documentation

No documentation available.

Content Model

%Property; %Proposition; %Justification;

Source

<element name="JustifiedProperty" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Property"/>
      <ref name="Proposition"/>
      <ref name="Justification"/>
    </element>

Element: JustifiedTheorem

Table 66. Element: JustifiedTheorem

Documentation

No documentation available.

Content Model

%Proposition; %Justification;

Source

<element name="JustifiedTheorem" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Proposition"/>
      <ref name="Justification"/>
    </element>

Element: LambdaVar

Table 67. Element: LambdaVar

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="LambdaVar" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
    </element>

Element: Let

Table 68. Element: Let

Documentation

No documentation available.

Content Model

( %Typ; )+

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="Let" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <oneOrMore>
        <ref name="Typ"/>
      </oneOrMore>
    </element>

Element: LocusVar

Table 69. Element: LocusVar

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="LocusVar" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
    </element>

Element: Not

Table 70. Element: Not

Documentation

No documentation available.

Content Model

%Formula;

Source

<element name="Not" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Formula"/>
    </element>

Element: NotationBlock

Table 71. Element: NotationBlock

Documentation

No documentation available.

Content Model

( ( %Let; | %AuxiliaryItem; ) )* %EndPosition;

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="NotationBlock" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <zeroOrMore>
        <choice>
          <ref name="Let"/>
          <ref name="AuxiliaryItem"/>
        </choice>
      </zeroOrMore>
      <ref name="EndPosition"/>
    </element>

Element: Notations

Table 72. Element: Notations

Documentation

No documentation available.

Content Model

%Signature; %Vocabularies; ? , ( %Pattern; )*

Attributes

Attribute

Type

Use

Documentation

aid xsd:stringOptional

Source

<element name="Notations" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="aid">
          <data type="string"/>
        </attribute>
      </optional>
      <optional>
        <ref name="Signature"/>
        <ref name="Vocabularies"/>
      </optional>
      <zeroOrMore>
        <ref name="Pattern"/>
      </zeroOrMore>
    </element>

Element: Now

Table 73. Element: Now

Documentation

No documentation available.

Content Model

%Reasoning; %BlockThesis;

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="Now" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <ref name="Position"/>
      <ref name="Reasoning"/>
      <ref name="BlockThesis"/>
    </element>

Element: Num

Table 74. Element: Num

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="Num" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
    </element>

Element: Pair

Table 75. Element: Pair

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

x xsd:integerOptional

y xsd:integerOptional

Source

<element name="Pair" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="x">
        <data type="integer"/>
      </attribute>
      <attribute name="y">
        <data type="integer"/>
      </attribute>
    </element>

Element: PartialDef

Table 76. Element: PartialDef

Documentation

No documentation available.

Content Model

( %Formula; | %Term; ) %Formula;

Source

<element name="PartialDef" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
          <choice>
            <ref name="Formula"/>
            <ref name="Term"/>
          </choice>
          <ref name="Formula"/>
        </element>

Element: Pattern

Table 77. Element: Pattern

Documentation

No documentation available.

Content Model

( | %Format; ) %ArgTypes;, Visible, Expansion ?

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "M" | "L" | "V" | "R" | "K" | "U" | "G" | "J" Optional

formatnr xsd:integerOptional

constrkind Enumeration: "M" | "L" | "V" | "R" | "K" | "U" | "G" | "J" Optional

constrnr xsd:integerOptional

antonymic xsd:booleanOptional

Source

<element name="Pattern" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="kind">
        <choice>
          <value>M</value>
          <value>L</value>
          <value>V</value>
          <value>R</value>
          <value>K</value>
          <value>U</value>
          <value>G</value>
          <value>J</value>
        </choice>
      </attribute>
      <choice>
        <attribute name="formatnr">
          <data type="integer"/>
        </attribute>
        <ref name="Format"/>
      </choice>
      <attribute name="constrkind">
        <choice>
          <value>M</value>
          <value>L</value>
          <value>V</value>
          <value>R</value>
          <value>K</value>
          <value>U</value>
          <value>G</value>
          <value>J</value>
        </choice>
      </attribute>
      <attribute name="constrnr">
        <data type="integer"/>
      </attribute>
      <optional>
        <attribute name="antonymic">
          <data type="boolean"/>
        </attribute>
      </optional>
      <ref name="ArgTypes"/>
      <element name="Visible">
        <zeroOrMore>
          <ref name="Int"/>
        </zeroOrMore>
      </element>
      <optional>
        <element name="Expansion">
          <ref name="Typ"/>
        </element>
      </optional>
    </element>

Element: PerCases

Table 78. Element: PerCases

Documentation

No documentation available.

Content Model

%Proposition; %Inference;

Source

<element name="PerCases" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Proposition"/>
      <ref name="Inference"/>
    </element>

Element: PerCasesReasoning

Table 79. Element: PerCasesReasoning

Documentation

No documentation available.

Content Model

( ( %BlockThesis; ( ( %CaseBlock; )+ | ( %SupposeBlock; )+ ) %PerCases; %Thesis; %EndPosition; ) | ( ( ( %CaseBlock; )+ | ( %SupposeBlock; )+ ) %PerCases; %EndPosition; %BlockThesis; ) )

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="PerCasesReasoning" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <choice>
        <group>
          <ref name="BlockThesis"/>
          <choice>
            <oneOrMore>
              <ref name="CaseBlock"/>
            </oneOrMore>
            <oneOrMore>
              <ref name="SupposeBlock"/>
            </oneOrMore>
          </choice>
          <ref name="PerCases"/>
          <ref name="Thesis"/>
          <ref name="EndPosition"/>
        </group>
        <group>
          <choice>
            <oneOrMore>
              <ref name="CaseBlock"/>
            </oneOrMore>
            <oneOrMore>
              <ref name="SupposeBlock"/>
            </oneOrMore>
          </choice>
          <ref name="PerCases"/>
          <ref name="EndPosition"/>
          <ref name="BlockThesis"/>
        </group>
      </choice>
    </element>

Element: Pred

Table 80. Element: Pred

Documentation

No documentation available.

Content Model

( %Term; )*

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "P" | "V" | "R" Optional

nr xsd:integerOptional

Source

<element name="Pred" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="kind">
        <choice>
          <value>P</value>
          <value>V</value>
          <value>R</value>
        </choice>
      </attribute>
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <zeroOrMore>
        <ref name="Term"/>
      </zeroOrMore>
    </element>

Element: Priority

Table 81. Element: Priority

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "O" | "K" | "L" Optional

symbolnr xsd:integerOptional

value xsd:integerOptional

Source

<element name="Priority" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
          <attribute name="kind">
            <choice>
              <value>O</value>
              <value>K</value>
              <value>L</value>
            </choice>
          </attribute>
          <attribute name="symbolnr">
            <data type="integer"/>
          </attribute>
          <attribute name="value">
            <data type="integer"/>
          </attribute>
        </element>

Element: PrivFunc

Table 82. Element: PrivFunc

Documentation

No documentation available.

Content Model

( %Term; )+

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="PrivFunc" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <oneOrMore>
        <ref name="Term"/>
      </oneOrMore>
    </element>

Element: PrivPred

Table 83. Element: PrivPred

Documentation

No documentation available.

Content Model

( %Term; )* %Formula;

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="PrivPred" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <zeroOrMore>
        <ref name="Term"/>
      </zeroOrMore>
      <ref name="Formula"/>
    </element>

Element: Projectivity

Table 84. Element: Projectivity

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Projectivity" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Proof

Table 85. Element: Proof

Documentation

No documentation available.

Content Model

%BlockThesis; %Reasoning;

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="Proof" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <ref name="Position"/>
      <ref name="BlockThesis"/>
      <ref name="Reasoning"/>
    </element>

Element: Properties

Table 86. Element: Properties

Documentation

No documentation available.

Content Model

( %Property; )+

Attributes

Attribute

Type

Use

Documentation

propertyarg1 xsd:integerOptional

propertyarg2 xsd:integerOptional

Source

<element name="Properties" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="propertyarg1">
        <data type="integer"/>
      </attribute>
      <attribute name="propertyarg2">
        <data type="integer"/>
      </attribute>
      <oneOrMore>
        <ref name="Property"/>
      </oneOrMore>
    </element>

Element: Proposition

Table 87. Element: Proposition

Documentation

No documentation available.

Content Model

%Formula;

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

nr xsd:integerOptional

Source

<element name="Proposition" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <ref name="Formula"/>
    </element>

Element: QuaTrm

Table 88. Element: QuaTrm

Documentation

No documentation available.

Content Model

%Term; %Typ;

Source

<element name="QuaTrm" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Term"/>
      <ref name="Typ"/>
    </element>

Element: RCluster

Table 89. Element: RCluster

Documentation

No documentation available.

Content Model

( %ErrorCluster; | ( %ArgTypes; %Typ; %Cluster; ) )

Source

<element name="RCluster" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="ErrorCluster"/>
        <group>
          <ref name="ArgTypes"/>
          <ref name="Typ"/>
          <ref name="Cluster"/>
        </group>
      </choice>
    </element>

Element: Reconsider

Table 90. Element: Reconsider

Documentation

No documentation available.

Content Model

%Typ;, ( %Term; )+ %Proposition; %Justification;

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="Reconsider" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <ref name="Typ"/>
      <oneOrMore>
        <ref name="Term"/>
      </oneOrMore>
      <ref name="Proposition"/>
      <ref name="Justification"/>
    </element>

Element: Ref

Table 91. Element: Ref

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

articlenr xsd:integerOptional

kind Enumeration: "T" | "D" Optional

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="Ref" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <optional>
        <attribute name="articlenr">
          <data type="integer"/>
        </attribute>
        <attribute name="kind">
          <choice>
            <value>T</value>
            <value>D</value>
          </choice>
        </attribute>
      </optional>
      <ref name="Position"/>
    </element>

Element: Reflexivity

Table 92. Element: Reflexivity

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Reflexivity" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Registration

Table 93. Element: Registration

Documentation

No documentation available.

Content Model

( %RCluster; | %FCluster; | %CCluster; ) ( %CorrectnessCondition; )* , %Correctness; ?

Source

<element name="Registration" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="RCluster"/>
        <ref name="FCluster"/>
        <ref name="CCluster"/>
      </choice>
      <zeroOrMore>
        <ref name="CorrectnessCondition"/>
      </zeroOrMore>
      <optional>
        <ref name="Correctness"/>
      </optional>
    </element>

Element: RegistrationBlock

Table 94. Element: RegistrationBlock

Documentation

No documentation available.

Content Model

( ( %Let; | %AuxiliaryItem; | %Registration; | %Canceled; ) )+ %EndPosition;

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="RegistrationBlock" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <oneOrMore>
        <choice>
          <ref name="Let"/>
          <ref name="AuxiliaryItem"/>
          <ref name="Registration"/>
          <ref name="Canceled"/>
        </choice>
      </oneOrMore>
      <ref name="EndPosition"/>
    </element>

Element: Registrations

Table 95. Element: Registrations

Documentation

No documentation available.

Content Model

%Signature; ? , ( ( %RCluster; | %CCluster; | %FCluster; ) )*

Attributes

Attribute

Type

Use

Documentation

aid xsd:stringOptional

Source

<element name="Registrations" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="aid">
          <data type="string"/>
        </attribute>
      </optional>
      <optional>
        <ref name="Signature"/>
      </optional>
      <zeroOrMore>
        <choice>
          <ref name="RCluster"/>
          <ref name="CCluster"/>
          <ref name="FCluster"/>
        </choice>
      </zeroOrMore>
    </element>

Element: Requirement

Table 96. Element: Requirement

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

constrkind Enumeration: "M" | "L" | "V" | "R" | "K" | "U" | "G" Optional

constrnr xsd:integerOptional

nr xsd:integerOptional

Source

<element name="Requirement" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
          <attribute name="constrkind">
            <choice>
              <value>M</value>
              <value>L</value>
              <value>V</value>
              <value>R</value>
              <value>K</value>
              <value>U</value>
              <value>G</value>
            </choice>
          </attribute>
          <attribute name="constrnr">
            <data type="integer"/>
          </attribute>
          <attribute name="nr">
            <data type="integer"/>
          </attribute>
        </element>

Element: Requirements

Table 97. Element: Requirements

Documentation

No documentation available.

Content Model

%Signature;, ( Requirement )*

Source

<element name="Requirements" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Signature"/>
      <zeroOrMore>
        <element name="Requirement">
          <attribute name="constrkind">
            <choice>
              <value>M</value>
              <value>L</value>
              <value>V</value>
              <value>R</value>
              <value>K</value>
              <value>U</value>
              <value>G</value>
            </choice>
          </attribute>
          <attribute name="constrnr">
            <data type="integer"/>
          </attribute>
          <attribute name="nr">
            <data type="integer"/>
          </attribute>
        </element>
      </zeroOrMore>
    </element>

Element: Reservation

Table 98. Element: Reservation

Documentation

No documentation available.

Content Model

%Typ;

Source

<element name="Reservation" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Typ"/>
    </element>

Element: Scheme

Table 99. Element: Scheme

Documentation

No documentation available.

Content Model

%ArgTypes;, %Formula;, ( %Formula; )*

Attributes

Attribute

Type

Use

Documentation

articlenr xsd:integerOptional

nr xsd:integerOptional

aid xsd:stringOptional

Source

<element name="Scheme" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="articlenr">
          <data type="integer"/>
        </attribute>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <optional>
        <attribute name="aid">
          <data type="string"/>
        </attribute>
      </optional>
      <ref name="ArgTypes"/>
      <ref name="Formula"/>
      <zeroOrMore>
        <ref name="Formula"/>
      </zeroOrMore>
    </element>

Element: SchemeBlock

Table 100. Element: SchemeBlock

Documentation

No documentation available.

Content Model

( ( %SchemeFuncDecl; | %SchemePredDecl; ) )* , SchemePremises %Proposition; %Justification; %EndPosition;

Attributes

Attribute

Type

Use

Documentation

schemenr xsd:integerOptional

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="SchemeBlock" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="schemenr">
        <data type="integer"/>
      </attribute>
      <ref name="Position"/>
      <zeroOrMore>
        <choice>
          <ref name="SchemeFuncDecl"/>
          <ref name="SchemePredDecl"/>
        </choice>
      </zeroOrMore>
      <element name="SchemePremises">
        <zeroOrMore>
          <ref name="Proposition"/>
        </zeroOrMore>
      </element>
      <ref name="Proposition"/>
      <ref name="Justification"/>
      <ref name="EndPosition"/>
    </element>

Element: SchemeFuncDecl

Table 101. Element: SchemeFuncDecl

Documentation

No documentation available.

Content Model

%ArgTypes; %Typ;

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="SchemeFuncDecl" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <ref name="ArgTypes"/>
      <ref name="Typ"/>
    </element>

Element: SchemePredDecl

Table 102. Element: SchemePredDecl

Documentation

No documentation available.

Content Model

%ArgTypes;

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="SchemePredDecl" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
      <ref name="ArgTypes"/>
    </element>

Element: SchemePremises

Table 103. Element: SchemePremises

Documentation

No documentation available.

Content Model

( %Proposition; )*

Source

<element name="SchemePremises" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <zeroOrMore>
          <ref name="Proposition"/>
        </zeroOrMore>
      </element>

Element: Schemes

Table 104. Element: Schemes

Documentation

No documentation available.

Content Model

%Signature; ? , ( %Scheme; )*

Attributes

Attribute

Type

Use

Documentation

aid xsd:stringOptional

Source

<element name="Schemes" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="aid">
          <data type="string"/>
        </attribute>
      </optional>
      <optional>
        <ref name="Signature"/>
      </optional>
      <zeroOrMore>
        <ref name="Scheme"/>
      </zeroOrMore>
    </element>

Element: Set

Table 105. Element: Set

Documentation

No documentation available.

Content Model

%Term; %Typ;

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="Set" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <ref name="Term"/>
      <ref name="Typ"/>
    </element>

Element: Signature

Table 106. Element: Signature

Documentation

No documentation available.

Content Model

( %ArticleID; )*

Source

<element name="Signature" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="ArticleID"/>
      </zeroOrMore>
    </element>

Element: SignatureWithCounts

Table 107. Element: SignatureWithCounts

Documentation

No documentation available.

Content Model

( %ConstrCounts; )*

Source

<element name="SignatureWithCounts" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
            <zeroOrMore>
              <ref name="ConstrCounts"/>
            </zeroOrMore>
          </element>

Element: SkippedProof

Table 108. Element: SkippedProof

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="SkippedProof" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <empty/>
    </element>

Element: StructLoci

Table 109. Element: StructLoci

Documentation

No documentation available.

Content Model

( %Pair; )*

Source

<element name="StructLoci" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="Pair"/>
      </zeroOrMore>
    </element>

Element: Suppose

Table 110. Element: Suppose

Documentation

No documentation available.

Content Model

( %Proposition; )+

Source

<element name="Suppose" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <oneOrMore>
        <ref name="Proposition"/>
      </oneOrMore>
    </element>

Element: SupposeBlock

Table 111. Element: SupposeBlock

Documentation

No documentation available.

Content Model

( ( %BlockThesis; %Suppose; %Thesis; %Reasoning; ) | ( %Suppose; %Reasoning; %BlockThesis; ) )

Attributes

Attribute

Type

Use

Documentation

line xsd:integerOptional

col xsd:integerOptional

Source

<element name="SupposeBlock" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Position"/>
      <choice>
        <group>
          <ref name="BlockThesis"/>
          <ref name="Suppose"/>
          <ref name="Thesis"/>
          <ref name="Reasoning"/>
        </group>
        <group>
          <ref name="Suppose"/>
          <ref name="Reasoning"/>
          <ref name="BlockThesis"/>
        </group>
      </choice>
    </element>

Element: Symbol

Table 112. Element: Symbol

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

kind xsd:stringOptional

nr xsd:integerOptional

name xsd:integerOptional

Source

<element name="Symbol" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
          <attribute name="kind">
            <data type="string"/>
          </attribute>
          <attribute name="nr">
            <data type="integer"/>
          </attribute>
          <attribute name="name">
            <data type="integer"/>
          </attribute>
        </element>

Element: SymbolCount

Table 113. Element: SymbolCount

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "G" | "K" | "L" | "M" | "O" | "R" | "U" | "V" Optional

nr xsd:integerOptional

Source

<element name="SymbolCount" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
              <attribute name="kind">
                <choice>
                  <value>G</value>
                  <value>K</value>
                  <value>L</value>
                  <value>M</value>
                  <value>O</value>
                  <value>R</value>
                  <value>U</value>
                  <value>V</value>
                </choice>
              </attribute>
              <attribute name="nr">
                <data type="integer"/>
              </attribute>
            </element>

Element: Symbols

Table 114. Element: Symbols

Documentation

No documentation available.

Content Model

( Symbol )*

Source

<element name="Symbols" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <element name="Symbol">
          <attribute name="kind">
            <data type="string"/>
          </attribute>
          <attribute name="nr">
            <data type="integer"/>
          </attribute>
          <attribute name="name">
            <data type="integer"/>
          </attribute>
        </element>
      </zeroOrMore>
    </element>

Element: Symmetry

Table 115. Element: Symmetry

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Symmetry" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Take

Table 116. Element: Take

Documentation

No documentation available.

Content Model

%Term;

Source

<element name="Take" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Term"/>
    </element>

Element: TakeAsVar

Table 117. Element: TakeAsVar

Documentation

No documentation available.

Content Model

%Typ; %Term;

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="TakeAsVar" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <ref name="Typ"/>
      <ref name="Term"/>
    </element>

Element: Theorem

Table 118. Element: Theorem

Documentation

No documentation available.

Content Model

%Formula;

Attributes

Attribute

Type

Use

Documentation

articlenr xsd:integerOptional

nr xsd:integerOptional

aid xsd:stringOptional

kind Enumeration: "T" | "D" Optional

Source

<element name="Theorem" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
          <optional>
            <attribute name="articlenr">
              <data type="integer"/>
            </attribute>
            <attribute name="nr">
              <data type="integer"/>
            </attribute>
          </optional>
          <optional>
            <attribute name="aid">
              <data type="string"/>
            </attribute>
          </optional>
          <attribute name="kind">
            <choice>
              <value>T</value>
              <value>D</value>
            </choice>
          </attribute>
          <ref name="Formula"/>
        </element>

Element: Theorems

Table 119. Element: Theorems

Documentation

No documentation available.

Content Model

%Signature; ? , ( Theorem )*

Attributes

Attribute

Type

Use

Documentation

aid xsd:stringOptional

Source

<element name="Theorems" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <optional>
        <attribute name="aid">
          <data type="string"/>
        </attribute>
      </optional>
      <optional>
        <ref name="Signature"/>
      </optional>
      <zeroOrMore>
        <element name="Theorem">
          <optional>
            <attribute name="articlenr">
              <data type="integer"/>
            </attribute>
            <attribute name="nr">
              <data type="integer"/>
            </attribute>
          </optional>
          <optional>
            <attribute name="aid">
              <data type="string"/>
            </attribute>
          </optional>
          <attribute name="kind">
            <choice>
              <value>T</value>
              <value>D</value>
            </choice>
          </attribute>
          <ref name="Formula"/>
        </element>
      </zeroOrMore>
    </element>

Element: Thesis

Table 120. Element: Thesis

Documentation

No documentation available.

Content Model

%Formula; %ThesisExpansions;

Source

<element name="Thesis" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <ref name="Formula"/>
      <ref name="ThesisExpansions"/>
    </element>

Element: ThesisExpansions

Table 121. Element: ThesisExpansions

Documentation

No documentation available.

Content Model

( %Pair; )*

Source

<element name="ThesisExpansions" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <ref name="Pair"/>
      </zeroOrMore>
    </element>

Element: Transitivity

Table 122. Element: Transitivity

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Transitivity" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Typ

Table 123. Element: Typ

Documentation

No documentation available.

Content Model

( %Cluster; )* , ( %Term; )*

Attributes

Attribute

Type

Use

Documentation

kind Enumeration: "M" | "G" | "errortyp" Optional

nr xsd:integerOptional

Source

<element name="Typ" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="kind">
        <choice>
          <value>M</value>
          <value>G</value>
          <value>errortyp</value>
        </choice>
      </attribute>
      <optional>
        <attribute name="nr">
          <data type="integer"/>
        </attribute>
      </optional>
      <zeroOrMore>
        <ref name="Cluster"/>
      </zeroOrMore>
      <zeroOrMore>
        <ref name="Term"/>
      </zeroOrMore>
    </element>

Element: UnexpectedProp

Table 124. Element: UnexpectedProp

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="UnexpectedProp" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <empty/>
      </element>

Element: Uniqueness

Table 125. Element: Uniqueness

Documentation

No documentation available.

Content Model

( %Formula; | ( %Proposition; %Justification; ) )

Source

<element name="Uniqueness" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="Formula"/>
        <group>
          <ref name="Proposition"/>
          <ref name="Justification"/>
        </group>
      </choice>
    </element>

Element: UnknownCorrCond

Table 126. Element: UnknownCorrCond

Documentation

No documentation available.

Content Model

( %Formula; | ( %Proposition; %Justification; ) )

Source

<element name="UnknownCorrCond" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <choice>
        <ref name="Formula"/>
        <group>
          <ref name="Proposition"/>
          <ref name="Justification"/>
        </group>
      </choice>
    </element>

Element: Var

Table 127. Element: Var

Documentation

No documentation available.

Content Model

Attributes

Attribute

Type

Use

Documentation

nr xsd:integerOptional

Source

<element name="Var" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <attribute name="nr">
        <data type="integer"/>
      </attribute>
    </element>

Element: Verum

Table 128. Element: Verum

Documentation

No documentation available.

Content Model

EMPTY

Source

<element name="Verum" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <empty/>
    </element>

Element: Visible

Table 129. Element: Visible

Documentation

No documentation available.

Content Model

( %Int; )*

Source

<element name="Visible" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
        <zeroOrMore>
          <ref name="Int"/>
        </zeroOrMore>
      </element>

Element: Vocabularies

Table 130. Element: Vocabularies

Documentation

No documentation available.

Content Model

( Vocabulary )*

Source

<element name="Vocabularies" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
      <zeroOrMore>
        <element name="Vocabulary">
          <ref name="ArticleID"/>
          <zeroOrMore>
            <element name="SymbolCount">
              <attribute name="kind">
                <choice>
                  <value>G</value>
                  <value>K</value>
                  <value>L</value>
                  <value>M</value>
                  <value>O</value>
                  <value>R</value>
                  <value>U</value>
                  <value>V</value>
                </choice>
              </attribute>
              <attribute name="nr">
                <data type="integer"/>
              </attribute>
            </element>
          </zeroOrMore>
        </element>
      </zeroOrMore>
    </element>

Element: Vocabulary

Table 131. Element: Vocabulary

Documentation

No documentation available.

Content Model

%ArticleID;, ( SymbolCount )*

Source

<element name="Vocabulary" xmlns:a="http://relaxng.org/ns/compatibility/annotations/1.0" xmlns="http://relaxng.org/ns/structure/1.0">
          <ref name="ArticleID"/>
          <zeroOrMore>
            <element name="SymbolCount">
              <attribute name="kind">
                <choice>
                  <value>G</value>
                  <value>K</value>
                  <value>L</value>
                  <value>M</value>
                  <value>O</value>
                  <value>R</value>
                  <value>U</value>
                  <value>V</value>
                </choice>
              </attribute>
              <attribute name="nr">
                <data type="integer"/>
              </attribute>
            </element>
          </zeroOrMore>
        </element>

Pattern: Adjective

Table 132. Pattern: Adjective

Namespace

Documentation

Adjective is a possibly negated (and paramaterized) attribute

Content Model

Adjective

Pattern: And

Table 133. Pattern: And

Namespace

Documentation

Conjunctive formula

Content Model

And

Pattern: ArgTypes

Table 134. Pattern: ArgTypes

Namespace

Documentation

Argument types of constructors, patterns, clusters, etc.

Content Model

ArgTypes

Pattern: Article

Table 135. Pattern: Article

Namespace

Documentation

The complete article after analyzer. aid specifies its name in uppercase.

Content Model

Article

Pattern: ArticleID

Table 136. Pattern: ArticleID

Namespace

Documentation

This is now only the unique name of an article.

Content Model

ArticleID

Pattern: Assume

Table 137. Pattern: Assume

Namespace

Documentation

One assumption may consist of several propositions.

Content Model

Assume

Pattern: AuxiliaryItem

Table 138. Pattern: AuxiliaryItem

Namespace

Documentation

Auxiliary items are items which do not change thesis.

Content Model

( %JustifiedProposition; | %Consider; | %Set; | %Reconsider; | %DefFunc; | %DefPred; )

Pattern: BlockThesis

Table 139. Pattern: BlockThesis

Namespace

Documentation

The block thesis is printed for proofs in the beginning and for diffuse reasoning in the end.

Content Model

BlockThesis

Pattern: By

Table 140. Pattern: By

Namespace

Documentation

By encodes one simple justification.

Content Model

By

Pattern: CCluster

Table 141. Pattern: CCluster

Namespace

Documentation

Conditional cluster. This says that Typ with the first cluster has also the second.

Content Model

CCluster

Pattern: Canceled

Table 142. Pattern: Canceled

Namespace

Documentation

Canceled theorem ( if on top-level), definition or registration (if inside such blocks). We should add to this the number of canceled items as an attribute.

Content Model

Canceled

Pattern: Case

Table 143. Pattern: Case

Namespace

Documentation

Case of one or more propositions.

Content Model

Case

Pattern: CaseBlock

Table 144. Pattern: CaseBlock

Namespace

Documentation

Block starting with one case, the direct and diffuse version (this depends on the kind of its parent block). The block thesis is printed for proofs in the beginning and for diffuse reasoning in the end.

Content Model

CaseBlock

Pattern: Cluster

Table 145. Pattern: Cluster

Namespace

Documentation

Cluster of adjectives

Content Model

Cluster

Pattern: Coherence

Table 146. Pattern: Coherence

Namespace

Documentation

No documentation available.

Content Model

Coherence

Pattern: Compatibility

Table 147. Pattern: Compatibility

Namespace

Documentation

No documentation available.

Content Model

Compatibility

Pattern: Conclusion

Table 148. Pattern: Conclusion

Namespace

Documentation

Justified conclusion. In text, this can appear as _hence_, _thus_ or _hereby_ (which starts diffuse conclusion).

Content Model

Conclusion

Pattern: Consider

Table 149. Pattern: Consider

Namespace

Documentation

First comes the reconstructed existential statement and its justification, then the new local constants and zero or more propositions about them. For easier presentation, nr optionally contains the number of the first local constant created here.

Content Model

Consider

Pattern: Consistency

Table 150. Pattern: Consistency

Namespace

Documentation

No documentation available.

Content Model

Consistency

Pattern: Const

Table 151. Pattern: Const

Namespace

Documentation

Normal local constant introduced e.g. by Let or Consider

Content Model

Const

Pattern: ConstrCounts

Table 152. Pattern: ConstrCounts

Namespace

Documentation

Constructor counts are used probably for renumerating. The article named can be given if not implicit. This implementation might change in some time.

Content Model

ConstrCounts

Pattern: Constructor

Table 153. Pattern: Constructor

Namespace

Documentation

Constructors are functors, predicates, attributes, etc. nr, kind and aid (article id) determine the constructor absolutely in MML, relnr optionally gives its serial number in environment for a particular article (it is not in prels). All have (possibly empty) properties, argtypes and some have one or more mother types. The optional final NatFunc are fields for agrregates and structmodes. aggregbase is for aggregates (maybe OVER-arguments), structmodeaggrnr is for structmodes (nr of corresponding aggregate)

Content Model

Constructor

Pattern: Constructors

Table 154. Pattern: Constructors

Namespace

Documentation

Constructors, either imported from other articles ( after accommodation) - the signature is implicit in that case, or exported from the current article - then the signature has to be specified. aid optionally specifies its article's name in uppercase.

Content Model

Constructors

Pattern: Correctness

Table 155. Pattern: Correctness

Namespace

Documentation

This is a way how to state all correctness conditions in one keyword. The relevant conditions are computed by the analyzer and printed here, their conjunction has to be justified.

Content Model

Correctness

Pattern: CorrectnessCondition

Table 156. Pattern: CorrectnessCondition

Namespace

Documentation

The possible correctness conditions are following. They can either be only stated in the Correctness, which conjugates them and proves them all, or come separately as a proposition with a justification.

Content Model

( %UnknownCorrCond; | %Coherence; | %Compatibility; | %Consistency; | %Existence; | %Uniqueness; )

Pattern: DefFunc

Table 157. Pattern: DefFunc

Namespace

Documentation

Private functor. First come the types of arguments, then its definition and the result type.

Content Model

DefFunc

Pattern: DefMeaning

Table 158. Pattern: DefMeaning

Namespace

Documentation

DefMeaning consists of the formulas and terms defining a constructor. It can be either defined by _equals_ (terms) or by _means_ (formulas). It may contain several partial (case) definitions - first in them comes the definition (term or formula) valid in that case and second comes the case formula. The final term or formula specifies the default case, it is mandatory if no partial definitions are given. If no default is given, the disjunction of all case formulas must be true (this have to be proved using the _consistency_ condition).

Content Model

DefMeaning

Pattern: DefPred

Table 159. Pattern: DefPred

Namespace

Documentation

Private predicate. First come the types of arguments, then its definition.

Content Model

DefPred

Pattern: DefTheorem

Table 160. Pattern: DefTheorem

Namespace

Documentation

Theorems created from definitions are now printed as separate top-level items after definitional blocks,

Content Model

DefTheorem

Pattern: Definiens

Table 161. Pattern: Definiens

Namespace

Documentation

Definiens of a constructor. This overlaps a bit with Constructor. First come the argument types and possibly also the result type. The optional formula is conjunction of all assumptions if any given. If this is a redefinition, essentials are indeces of arguments corresponding to the arguments of original, otherwise it is just identity. This could be now encode with just one number like the superfluous does for Constructor.

Content Model

Definiens

Pattern: Definientia

Table 162. Pattern: Definientia

Namespace

Documentation

Definientia, either imported from other articles ( after accommodation) - the signature is implicit in that case, or exported from the current article - then the signature has to be specified. aid optionally specifies article's name in uppercase.

Content Model

Definientia

Pattern: Definition

Table 163. Pattern: Definition

Namespace

Documentation

Definition of a functor, predicate, mode, attribute or structure. with optional label, properties and correctness conditions. Sometimes no constructor is created (e.g. for expandable modes). The second optional form creating three or more constructors is for structure definitions, which define the aggregate functor, the structure mode, the strict attribute and zero or more selectors. If any definientia and definitional theorems are created, they follow immediately after the enclosing definitional block (this might be changed in the future).

Content Model

Definition

Pattern: DefinitionBlock

Table 164. Pattern: DefinitionBlock

Namespace

Documentation

A block of one or more (possibly canceled) (re)definitions, possibly with assumptions. If any definientia and definitional theorems are created, they follow immediately after this block.

Content Model

DefinitionBlock

Pattern: EndPosition

Table 165. Pattern: EndPosition

Namespace

Documentation

Ending position (e.g. of blocks).

Content Model

EndPosition

Pattern: ErrorCluster

Table 166. Pattern: ErrorCluster

Namespace

Documentation

This encodes error during cluster processing

Content Model

ErrorCluster

Pattern: ErrorFrm

Table 167. Pattern: ErrorFrm

Namespace

Documentation

Incorrect (erroneous formula) - e.g. containing undefined symbols

Content Model

ErrorFrm

Pattern: ErrorTrm

Table 168. Pattern: ErrorTrm

Namespace

Documentation

Incorrect (erroneous term) - e.g. containing undefined symbols

Content Model

ErrorTrm

Pattern: Existence

Table 169. Pattern: Existence

Namespace

Documentation

No documentation available.

Content Model

Existence

Pattern: FCluster

Table 170. Pattern: FCluster

Namespace

Documentation

Functor (term) cluster. This says that exists Term with Cluster.

Content Model

FCluster

Pattern: Fields

Table 171. Pattern: Fields

Namespace

Documentation

Specify numbers of fields of aggregates and structmodes.

Content Model

Fields

Pattern: For

Table 172. Pattern: For

Namespace

Documentation

Universally quantified formula

Content Model

For

Pattern: Format

Table 173. Pattern: Format

Namespace

Documentation

Format keeps the kind of a given symbol and arities. For bracket formats (K) this keeps both symbols. Optionally a nr (of the format) is kept, to which patterns may refer, This implementation might change in some time.

Content Model

Format

Pattern: Formats

Table 174. Pattern: Formats

Namespace

Documentation

Format info contains symbol formats and priorities. Priorities are used only for functor symbols. This implementation might change in some time.

Content Model

Formats

Pattern: Formula

Table 175. Pattern: Formula

Namespace

Documentation

No documentation available.

Content Model

( %Not; | %And; | %For; | %Pred; | %PrivPred; | %Is; | %Verum; | %ErrorFrm; )

Pattern: Fraenkel

Table 176. Pattern: Fraenkel

Namespace

Documentation

Fraenkel term is defined by the types of its lambda arguments, its lambda term and the separating formula.

Content Model

Fraenkel

Pattern: FreeVar

Table 177. Pattern: FreeVar

Namespace

Documentation

Free variable - used only internally in checker

Content Model

FreeVar

Pattern: From

Table 178. Pattern: From

Namespace

Documentation

From encodes one scheme justification, it cannot be linked.

Content Model

From

Pattern: Func

Table 179. Pattern: Func

Namespace

Documentation

Functor terms - schematic, aggregates, normal and selectors

Content Model

Func

Pattern: Given

Table 180. Pattern: Given

Namespace

Documentation

This is existential assumption, it may be used when the normal assumption starts with existential quantifier. In that case, the existential variables are introduced as local constants. For easier presentation, nr optionally contains the number of the first local constant created here.

Content Model

Given

Pattern: InfConst

Table 181. Pattern: InfConst

Namespace

Documentation

Inference constant - used for internal term sharing

Content Model

InfConst

Pattern: Inference

Table 182. Pattern: Inference

Namespace

Documentation

No documentation available.

Content Model

( %By; | %From; | ErrorInf )

Pattern: Int

Table 183. Pattern: Int

Namespace

Documentation

Single integer

Content Model

Int

Pattern: Is

Table 184. Pattern: Is

Namespace

Documentation

Qualification formula (claims that a term has certaing type)

Content Model

Is

Pattern: It

Table 185. Pattern: It

Namespace

Documentation

_It_ is a special term used in definitions. Probably no longer used on this level.

Content Model

It

Pattern: IterEquality

Table 186. Pattern: IterEquality

Namespace

Documentation

Iterative equality. The ptional number is label.

Content Model

IterEquality

Pattern: IterStep

Table 187. Pattern: IterStep

Namespace

Documentation

This is one step in an iterative equation.

Content Model

IterStep

Pattern: Justification

Table 188. Pattern: Justification

Namespace

Documentation

Direct justification.

Content Model

( %Inference; | %Proof; | %SkippedProof; )

Pattern: JustifiedProperty

Table 189. Pattern: JustifiedProperty

Namespace

Documentation

A property of a constructor, the proposition expreesing it, and its justification.

Content Model

JustifiedProperty

Pattern: JustifiedProposition

Table 190. Pattern: JustifiedProposition

Namespace

Documentation

No documentation available.

Content Model

( %Now; | %IterEquality; | ( %Proposition; %Justification; ) )

Pattern: JustifiedTheorem

Table 191. Pattern: JustifiedTheorem

Namespace

Documentation

Theorem as a proposition with justification.

Content Model

JustifiedTheorem

Pattern: LambdaVar

Table 192. Pattern: LambdaVar

Namespace

Documentation

Lambda variable - unused now

Content Model

LambdaVar

Pattern: Let

Table 193. Pattern: Let

Namespace

Documentation

Introduction of local constants, the numbering is automatic, so only types are needed. For easier presentation, nr optionally contains the number of the first local constant created here.

Content Model

Let

Pattern: LocusVar

Table 194. Pattern: LocusVar

Namespace

Documentation

Locus variable used usually for pattern matching. Their types are given elsewhere in data using them - see e.g. Constructor

Content Model

LocusVar

Pattern: Not

Table 195. Pattern: Not

Namespace

Documentation

Negation

Content Model

Not

Pattern: NotationBlock

Table 196. Pattern: NotationBlock

Namespace

Documentation

Block of synonyms or antonyms. The patterns are semantically irrelevant and are not printed yet - fix this.

Content Model

NotationBlock

Pattern: Notations

Table 197. Pattern: Notations

Namespace

Documentation

Notations, either imported from other articles ( after accommodation) - the signature is implicit in that case, or exported from the current article - then the signature and vocabularies have to be specified. aid optionally specifies article's name in uppercase.

Content Model

Notations

Pattern: Now

Table 198. Pattern: Now

Namespace

Documentation

Diffuse statement - its thesis is reconstructed in the end. Label (nr) of diffuse statement (if any) is label of its thesis.

Content Model

Now

Pattern: Num

Table 199. Pattern: Num

Namespace

Documentation

Numeral

Content Model

Num

Pattern: Pair

Table 200. Pattern: Pair

Namespace

Documentation

This is a pair of integers

Content Model

Pair

Pattern: Pattern

Table 201. Pattern: Pattern

Namespace

Documentation

Patterns map formats with argtypes to constructors. The format is either specified as a number (then it must be available in some table), or is given explicitely. Visible are indeces of visible (nonhidden) arguments. If antonymic, its constructor has to be negated. Mode patterns can have expansion instead of just a constructor - this might be done for other patterns too, or replaced by the _equals_ mechanism. The J (forgetful functor) patterns are actually an example of another expanded patterns, but the expansion is uniform for all of them, so it does not have to be given. The invalid ConstrKind J is now used for forgetful functors, this should be changed.

Content Model

Pattern

Pattern: PerCases

Table 202. Pattern: PerCases

Namespace

Documentation

This justifies the case split (the disjunction of all Suppose or Case items in direct subblocks) in PerCasesReasoning. The case split is only known after all subblocks are known, so this is the last item in its block, not like in the Mizar text.

Content Model

PerCases

Pattern: PerCasesReasoning

Table 203. Pattern: PerCasesReasoning

Namespace

Documentation

Reasoning per cases. It only contains CaseBlock or SupposeBlock subblocks, with the exception of the mandatory last PerCases justifying the case split. Direct and diffuse versions are possible (this depends on the kind of its parent block). The block thesis is printed for proofs in the beginning and for diffuse reasoning in the end.

Content Model

PerCasesReasoning

Pattern: Position

Table 204. Pattern: Position

Namespace

Documentation

No documentation available.

Attributes

Attribute

Type

Use

Documentation

line xsd:integerRequired

col xsd:integerRequired

Pattern: Pred

Table 205. Pattern: Pred

Namespace

Documentation

Atomic predicate formulas - schematic, attributive and normal

Content Model

Pred

Pattern: PrivFunc

Table 206. Pattern: PrivFunc

Namespace

Documentation

Private functor with arguments is a shorthand for another term. The first (mandatory) term is the expansion, arguments follow.

Content Model

PrivFunc

Pattern: PrivPred

Table 207. Pattern: PrivPred

Namespace

Documentation

Private predicate with arguments is a shorthand for another formula

Content Model

PrivPred

Pattern: Proof

Table 208. Pattern: Proof

Namespace

Documentation

Direct proof of some proposition (which is the proof's thesis). Label (nr) of proof (if any) is label of its thesis.

Content Model

Proof

Pattern: Properties

Table 209. Pattern: Properties

Namespace

Documentation

Properties of constructors; if some given, the first and the second argument to which they apply must be specified.

Content Model

Properties

Pattern: Property

Table 210. Pattern: Property

Namespace

Documentation

No documentation available.

Content Model

( UnexpectedProp | Symmetry | Reflexivity | Irreflexivity | Associativity | Transitivity | Commutativity | Connectedness | Antisymmetry | Idempotence | Involutiveness | Projectivity | Abstractness )

Pattern: Proposition

Table 211. Pattern: Proposition

Namespace

Documentation

Proposition is a sentence with position and possible label

Content Model

Proposition

Pattern: QuaTrm

Table 212. Pattern: QuaTrm

Namespace

Documentation

Qua terms capture the retyping term qua type construct, but they are probably no longer used on this level.

Content Model

QuaTrm

Pattern: RCluster

Table 213. Pattern: RCluster

Namespace

Documentation

Existential (registration) cluster. This says that exists Typ with Cluster.

Content Model

RCluster

Pattern: Reasoning

Table 214. Pattern: Reasoning

Namespace

Documentation

Reasoning is a series of skeleton and auxiliary items, finished by optional per cases reasoning.

Content Model

( ( %SkeletonItem; | %AuxiliaryItem; ) )* , %PerCasesReasoning; ? %EndPosition;

Pattern: Reconsider

Table 215. Pattern: Reconsider

Namespace

Documentation

First comes the target type, then the reconsidered terms. For all these terms a new local variable with the target type is created, and its equality to the corresponding term is remembered. Finally the proposition about the typing is given and justified. For easier presentation, nr optionally contains the number of the first local constant created here.

Content Model

Reconsider

Pattern: Ref

Table 216. Pattern: Ref

Namespace

Documentation

Reference can be either private (coming from the current article) - their number is the position at the stack of accessible references (so it is not unique), or library - these additionally contain their kind (theorem or definition) and article nr. The position in the inference is kept for error messaging.

Content Model

Ref

Pattern: Registration

Table 217. Pattern: Registration

Namespace

Documentation

One justified cluster registration. The correctness conditions could be made more specific for each.

Content Model

Registration

Pattern: RegistrationBlock

Table 218. Pattern: RegistrationBlock

Namespace

Documentation

Block of cluster registrations.

Content Model

RegistrationBlock

Pattern: Registrations

Table 219. Pattern: Registrations

Namespace

Documentation

Registrations, either imported from other articles ( after accommodation) - the signature is implicit in that case, or exported from the current article - then the signature has to be specified. aid optionally specifies its article's name in uppercase.

Content Model

Registrations

Pattern: Requirements

Table 220. Pattern: Requirements

Namespace

Documentation

Requirements (now only the exported form). The second number specifies the requirement - this could be changed to enumerated types for better understanding.

Content Model

Requirements

Pattern: Reservation

Table 221. Pattern: Reservation

Namespace

Documentation

Reservation of a new variable for a type.

Content Model

Reservation

Pattern: Scheme

Table 222. Pattern: Scheme

Namespace

Documentation

Schemes keep types of their second-order variables. First comes the scheme thesis, then the premises. The article number and order in article can be given, otherwise it belongs to the current article and order is implicit. Optional aid attribute specifies article name.

Content Model

Scheme

Pattern: SchemeBlock

Table 223. Pattern: SchemeBlock

Namespace

Documentation

Scheme blocks are used for declaring the types of second-order variables appearing in a scheme, and for its justification. This could be a bit unified with Scheme later.

Content Model

SchemeBlock

Pattern: SchemeFuncDecl

Table 224. Pattern: SchemeFuncDecl

Namespace

Documentation

Declaration of a scheme functor.

Content Model

SchemeFuncDecl

Pattern: SchemePredDecl

Table 225. Pattern: SchemePredDecl

Namespace

Documentation

Declaration of a scheme predicate.

Content Model

SchemePredDecl

Pattern: Schemes

Table 226. Pattern: Schemes

Namespace

Documentation

Schemes, either imported from other articles ( after accommodation) - the signature is implicit in that case, or exported from the current article - then the signature has to be specified. aid optionally specifies article's name in uppercase.

Content Model

Schemes

Pattern: Set

Table 227. Pattern: Set

Namespace

Documentation

This is e.g.: set a = f(b); . The type of the new local constant is given. This local constant is now always expanded to its definition, and should not directly appear in any expression, but it is now needed for some implementation reasons. For easier presentation, nr optionally contains the number of the first local constant created here.

Content Model

Set

Pattern: Signature

Table 228. Pattern: Signature

Namespace

Documentation

Signature is a list of articles from which we import constructors.

Content Model

Signature

Pattern: SkeletonItem

Table 229. Pattern: SkeletonItem

Namespace

Documentation

Skeleton items change the current thesis, for Proof the changed Thesis together with used expansions is printed explicitely after them. PerCasesReasoning is not included here.

Content Model

( %Let; | %Conclusion; | %Assume; | %Given; | %Take; | %TakeAsVar; ) %Thesis; ?

Pattern: SkippedProof

Table 230. Pattern: SkippedProof

Namespace

Documentation

This means that the author has skipped the proof. Articles with such items are not yet fully completed.

Content Model

SkippedProof

Pattern: StructLoci

Table 231. Pattern: StructLoci

Namespace

Documentation

Structural loci are not used yet (that is all I know about them).

Content Model

StructLoci

Pattern: Suppose

Table 232. Pattern: Suppose

Namespace

Documentation

Supposition of one or more propositions.

Content Model

Suppose

Pattern: SupposeBlock

Table 233. Pattern: SupposeBlock

Namespace

Documentation

Block starting with one supposition, the direct and diffuse version (this depends on the kind of its parent block). The block thesis is printed for proofs in the beginning and for diffuse reasoning in the end.

Content Model

SupposeBlock

Pattern: Symbols

Table 234. Pattern: Symbols

Namespace

Documentation

Local dictionary for an article. The symbol kinds still use very internal notation.

Content Model

Symbols

Attributes

Attribute

Type

Use

Documentation

aid xsd:stringOptional

Pattern: Take

Table 235. Pattern: Take

Namespace

Documentation

Take without equality. This does not introduce a new local constant, just changes the thesis.

Content Model

Take

Pattern: TakeAsVar

Table 236. Pattern: TakeAsVar

Namespace

Documentation

Take with equality. This introduces a new local constant, whose type is given here. For easier presentation, nr optionally contains the number of the first local constant created here.

Content Model

TakeAsVar

Pattern: Term

Table 237. Pattern: Term

Namespace

Documentation

No documentation available.

Content Model

( %Var; | %LocusVar; | %FreeVar; | %LambdaVar; | %Const; | %InfConst; | %Num; | %Func; | %PrivFunc; | %Fraenkel; | %QuaTrm; | %It; | %ErrorTrm; )

Pattern: Theorems

Table 238. Pattern: Theorems

Namespace

Documentation

Theorems, either imported from other articles ( after accommodation) - the signature is implicit in that case, or exported from the current article - then the signature has to be specified. They can be either ordinary or definitional. The article number and order in article can be given, otherwise it belongs to the current article and order is implicit. Optional aid attribute specifies article name.

Content Model

Theorems

Pattern: Thesis

Table 239. Pattern: Thesis

Namespace

Documentation

The changed thesis is printed after skeleton items in proofs, together with the numbers of definientia used for its expansion.

Content Model

Thesis

Pattern: ThesisExpansions

Table 240. Pattern: ThesisExpansions

Namespace

Documentation

Numbers of Definiens used in expanding the thesis, together with their counts.

Content Model

ThesisExpansions

Pattern: Typ

Table 241. Pattern: Typ

Namespace

Documentation

Parameterized type - either mode or structure First goes the LowerCluster, than UpperCluster

Content Model

Typ

Pattern: Uniqueness

Table 242. Pattern: Uniqueness

Namespace

Documentation

No documentation available.

Content Model

Uniqueness

Pattern: UnknownCorrCond

Table 243. Pattern: UnknownCorrCond

Namespace

Documentation

No documentation available.

Content Model

UnknownCorrCond

Pattern: Var

Table 244. Pattern: Var

Namespace

Documentation

Normal bound variable (deBruijn index). Their types are given in quantification - see For, Fraenkel

Content Model

Var

Pattern: Verum

Table 245. Pattern: Verum

Namespace

Documentation

Verum (true formula)

Content Model

Verum

Pattern: Vocabularies

Table 246. Pattern: Vocabularies

Namespace

Documentation

Vocabularies keep for each article its symbol numbers. This implementation might change in some time.

Content Model

Vocabularies