Introducing Euclidean Relations to Mizar

Total Page:16

File Type:pdf, Size:1020Kb

Introducing Euclidean Relations to Mizar Proceedings of the Federated Conference on DOI: 10.15439/2017F368 Computer Science and Information Systems pp. 245–248 ISSN 2300-5963 ACSIS, Vol. 11 Introducing Euclidean Relations to Mizar Adam Naumowicz, Artur Korniłowicz Institute of Informatics, University of Białystok ul. Ciołkowskiego 1 M, 15-245 Białystok, Poland Email: {adamn, arturk}@math.uwb.edu.pl Abstract—In this paper we present the methodology of imple- property has been analyzed and implemented most recently menting a new enhancement of the Mizar proof checker based on [15]. enabling special processing of Euclidean predicates, i.e. binary Table I presents how many registrations of predicate prop- predicates which fulfill a specific variant of transitivity postulated by Euclid. Typically, every proof step in formal mathematical erties are used in the MML. The data has been collected reasoning is associated with a formula to be proved and a list with Mizar Version 8.1.05 working with the MML Version of references used to justify the formula. With the proposed 5.37.1275.2 enhancement, the Euclidean property of given relations can be Property Occurrences Articles registered during their definition, and so the verification of some reflexivity 138 91 proof steps related to these relations can be automated to avoid irreflexivity 11 10 explicit referencing. symmetry 122 82 asymmetry 6 6 I. INTRODUCTION connectedness 4 4 total 281 119 HE Mizar system [1], [2], [3] is a computer proof- Table I T assistant system used for encoding formal mathematical PREDICATE PROPERTIES OCCURRENCES data (definitions and theorems) and verifying mathematical proofs. The system comprises a dedicated formal computer language – the Mizar language, a collection of command-line On the other hand, Table II shows the impact of registering tools including the VERIFIER and a repository of formal texts predicate properties for proofs stored in the library as the – Mizar Mathematical Library (MML) that have been written number of errors occurring after removing registrations of the in the Mizar language and machine-verified for their logical properties from texts, and the numbers of articles with such correctness by the VERIFIER. errors. The Mizar language preserves many features of natu- Property Errors Affected articles ral language mathematical writing. It is designed to write reflexivity 356 44 declarative-style documents both readable for humans and irreflexivity 9 2 effectively processed by computers.1 The feature-rich language symmetry 498 47 asymmetry 6 4 enables producing rigorous and semantically unambiguous connectedness 65 4 texts. Apart from rules for writing traditional mathematical total 934 73 items (e.g. definitions, lemmas, theorems, proof steps, etc.) Table II it also provides syntactic constructions to launch specialized PREDICATE PROPERTIES IMPACT algorithms for processing particular mechanisms (e.g. term identifications, term reductions [7], flexary connectives [8]) increasing computational power of VERIFIER (e.g. equational In this paper we propose strengthening the Mizar system calculus [9], [10]). There have also been experiments on using by implementing the representation of two new properties – 3 specialized external systems to increase computational power rightEuclidean and leftEuclidean. The properties of the Mizar system in selected domains [11], [12], [13]. are described in Section II. In Section III we present some Mizar allows registering various properties of predicates examples of Euclidean properties found in the current MML. and functors [14] when defining new notions. Let us briefly In Section IV we indicate several directions of further devel- recall that the set of currently implemented properties in- opment of processing properties in Mizar. cludes involutiveness and projectivity for unary II. THE EUCLIDEAN PROPERTY operations, as well as commutativity and idempotence An example of a property which does not have its corre- for binary operations. As far as binary predicates are con- sponding representation in Mizar yet is the Euclidean property. cerned, which is directly related to the topic of this pa- per, the current version of the Mizar system supports reg- 2Computations were carried out at the Computer Center of University of istering reflexivity, irreflexivity, symmetry, Białystok http://uco.uwb.edu.pl 3An experimental version of the VERIFIER executable file for the Linux asymmetry and connectedness. The transitivity platform implementing the new features as well as other supplementary resources required for it to work with the current MML are available at 1The legibility of proofs is a subject of ongoing research [4], [5], [6]. http://alioth.uwb.edu.pl/~artur/euclidean/euclidean_ver.zip. IEEE Catalog Number: CFP1785N-ART c 2017, PTI 245 246 PROCEEDINGS OF THE FEDCSIS. PRAGUE, 2017 This property appears, most notably, in the set of axiomatic It should be noted that the form of definitions and a corre- statements given at the start of Book I of Euclid’s The sponding correctness proof can in general be more complicated Elements [16] as Common Notion 1, which states that: Things when the definition has several cases. Below is a formal repre- which are equal to the same thing are also equal to each sentation of the correctness proof structure in the case of a def- 4 other. Formally speaking, a binary relation R on a set X is inition with three explicit cases (Γ1(x1, x2, . , xn, y1, y2), Euclidean (sometimes called right Euclidean) if it satisfies the Γ2(x1, x2, . , xn, y1, y2) and Γ3(x1, x2, . , xn, y1, y2)) as following condition: ∀a, b, c ∈ X (a R b ∧ a R c → b R c). well as the default case (introduced by otherwise): R X Dually, a relation on may be called left Euclidean if definition ∀a, b, c ∈ X (b R a ∧ c R a → b R c). let x1 be θ1, x2 be θ2, . , xn be θn, y1, y2 be θn+1; The property of being Euclidean is a variant of transitivity, pred π(y1, y2) means :ident: x , x , . , xn, y , y if x , x , . , xn, y , y , but the properties are indeed different. A transitive relation Φ1( 1 2 1 2) Γ1( 1 2 1 2) Φ2(x1, x2, . , xn, y1, y2) if Γ2(x1, x2, . , xn, y1, y2), is Euclidean only if it is also symmetric. Only a symmetric Φ3(x1, x2, . , xn, y1, y2) if Γ3(x1, x2, . , xn, y1, y2) Euclidean relation is transitive. A relation which is both otherwise Φn(x1, x2, . , xn, y1, y2); consistency; Euclidean and reflexive is also symmetric and therefore it is rightEuclidean an equivalence relation. proof In the sequel we describe an enhancement of the Mizar sys- thus for a, b, c being θn+1 st ( tem supporting automatic processing of Euclidean predicates. (Γ1(x1, x2, . , xn, a, b) implies Φ1(x1, x2, . , xn, a, b)) & The automation involves specific computations performed dur- (Γ2(x1, x2, . , xn, a, b) implies Φ2(x1, x2, . , xn, a, b)) & ing the verification process.5 (Γ3(x1, x2, . , xn, a, b) implies Φ3(x1, x2, . , xn, a, b)) & (not Γ1(x1, x2, . , xn, a, b) & To enable such an automation, when a new predicate is not Γ2(x1, x2, . , xn, a, b) & being defined, if it is Euclidean, it should be declared as such. not Γ3(x1, x2, . , xn, a, b) implies The declaration is placed within a definitional block with the Φn(x1, x2, . , xn, a, b)) & (Γ1(x1, x2, . , xn, a, c) implies Φ1(x1, x2, . , xn, a, c)) & following Mizar syntax for right Euclidean: (Γ2(x1, x2, . , xn, a, c) implies Φ2(x1, x2, . , xn, a, c)) & (Γ3(x1, x2, . , xn, a, c) implies Φ3(x1, x2, . , xn, a, c)) & definition (not Γ1(x1, x2, . , xn, a, c) & n n n let x1 be θ1, x2 be θ2, . , x be θ , y1, y2 be θ +1; not Γ2(x1, x2, . , xn, a, c) & ident pred π(y1, y2) means : : not Γ3(x1, x2, . , xn, a, c) implies n Φ(x1, x2, . , x , y1, y2); Φn(x1, x2, . , xn, a, c)) rightEuclidean ) holds proof ( , , n thus for a b c being θ +1 (Γ1(x1, x2, . , xn, b, c) implies Φ1(x1, x2, . , xn, b, c)) & n n st Φ(x1, x2, . , x , a, b) & Φ(x1, x2, . , x , a, c) (Γ2(x1, x2, . , xn, b, c) implies Φ2(x1, x2, . , xn, b, c)) & n holds Φ(x1, x2, . , x , b, c); (Γ3(x1, x2, . , xn, b, c) implies Φ3(x1, x2, . , xn, b, c)) & end; (not Γ1(x1, x2, . , xn, b, c) & end; not Γ2(x1, x2, . , xn, b, c) & not Γ3(x1, x2, . , xn, b, c) implies and left Euclidean, respectively: Φn(x1, x2, . , xn, b, c)) ); definition end; let x1 be θ1, x2 be θ2, . , xn be θn, y1, y2 be θn+1; end; pred π(y1, y2) means :ident: Φ(x1, x2, . , xn, y1, y2); The proof for a left Euclidean predicate with an analogous leftEuclidean proof set of conditions would look like this: thus for a, b, c being θn+1 definition st Φ(x1, x2, . , xn, b, a) & Φ(x1, x2, . , xn, c, a) let x be θ , x be θ , . , xn be θn, y , y be θn ; holds Φ(x1, x2, . , xn, b, c); 1 1 2 2 1 2 +1 ident end; pred π(y1, y2) means : : end; Φ1(x1, x2, . , xn, y1, y2) if Γ1(x1, x2, . , xn, y1, y2), Φ2(x1, x2, . , xn, y1, y2) if Γ2(x1, x2, . , xn, y1, y2), The statements of the formulas of correctness proofs shown Φ3(x1, x2, . , xn, y1, y2) if Γ3(x1, x2, . , xn, y1, y2) otherwise Φn(x1, x2, . , xn, y1, y2); in both the above definitions must be proved according to consistency; a special formula expressing the corresponding property of leftEuclidean the defined predicate. For example, having such a definition, proof thus for a, b, c being θn+1 st whenever VERIFIER meets a conjunction of formulas π(a, b) ( and π(a, c) within an inference, and the predicate π is known (Γ1(x1, x2, .
Recommended publications
  • Simple Laws About Nonprominent Properties of Binary Relations
    Simple Laws about Nonprominent Properties of Binary Relations Jochen Burghardt jochen.burghardt alumni.tu-berlin.de Nov 2018 Abstract We checked each binary relation on a 5-element set for a given set of properties, including usual ones like asymmetry and less known ones like Euclideanness. Using a poor man's Quine-McCluskey algorithm, we computed prime implicants of non-occurring property combinations, like \not irreflexive, but asymmetric". We considered the laws obtained this way, and manually proved them true for binary relations on arbitrary sets, thus contributing to the encyclopedic knowledge about less known properties. Keywords: Binary relation; Quine-McCluskey algorithm; Hypotheses generation arXiv:1806.05036v2 [math.LO] 20 Nov 2018 Contents 1 Introduction 4 2 Definitions 8 3 Reported law suggestions 10 4 Formal proofs of property laws 21 4.1 Co-reflexivity . 21 4.2 Reflexivity . 23 4.3 Irreflexivity . 24 4.4 Asymmetry . 24 4.5 Symmetry . 25 4.6 Quasi-transitivity . 26 4.7 Anti-transitivity . 28 4.8 Incomparability-transitivity . 28 4.9 Euclideanness . 33 4.10 Density . 38 4.11 Connex and semi-connex relations . 39 4.12 Seriality . 40 4.13 Uniqueness . 42 4.14 Semi-order property 1 . 43 4.15 Semi-order property 2 . 45 5 Examples 48 6 Implementation issues 62 6.1 Improved relation enumeration . 62 6.2 Quine-McCluskey implementation . 64 6.3 On finding \nice" laws . 66 7 References 69 List of Figures 1 Source code for transitivity check . .5 2 Source code to search for right Euclidean non-transitive relations . .5 3 Timing vs. universe cardinality .
    [Show full text]
  • Simple Laws About Nonprominent Properties of Binary Relations Jochen Burghardt
    Simple Laws about Nonprominent Properties of Binary Relations Jochen Burghardt To cite this version: Jochen Burghardt. Simple Laws about Nonprominent Properties of Binary Relations. 2018. hal- 02948115 HAL Id: hal-02948115 https://hal.archives-ouvertes.fr/hal-02948115 Preprint submitted on 24 Sep 2020 HAL is a multi-disciplinary open access L’archive ouverte pluridisciplinaire HAL, est archive for the deposit and dissemination of sci- destinée au dépôt et à la diffusion de documents entific research documents, whether they are pub- scientifiques de niveau recherche, publiés ou non, lished or not. The documents may come from émanant des établissements d’enseignement et de teaching and research institutions in France or recherche français ou étrangers, des laboratoires abroad, or from public or private research centers. publics ou privés. Simple Laws about Nonprominent Properties of Binary Relations Jochen Burghardt jochen.burghardt alumni.tu-berlin.de Nov 2018 Abstract We checked each binary relation on a 5-element set for a given set of properties, including usual ones like asymmetry and less known ones like Euclideanness. Using a poor man's Quine-McCluskey algorithm, we computed prime implicants of non-occurring property combinations, like \not irreflexive, but asymmetric". We considered the laws obtained this way, and manually proved them true for binary relations on arbitrary sets, thus contributing to the encyclopedic knowledge about less known properties. Keywords: Binary relation; Quine-McCluskey algorithm; Hypotheses generation Contents 1 Introduction 4 2 Definitions 8 3 Reported law suggestions 10 4 Formal proofs of property laws 21 4.1 Co-reflexivity . 21 4.2 Reflexivity . 23 4.3 Irreflexivity .
    [Show full text]
  • The Mathematical Landscape a Guided Tour
    Claremont Colleges Scholarship @ Claremont CMC Senior Theses CMC Student Scholarship 2011 The aM thematical Landscape Antonio Collazo Claremont McKenna College Recommended Citation Collazo, Antonio, "The aM thematical Landscape" (2011). CMC Senior Theses. Paper 116. http://scholarship.claremont.edu/cmc_theses/116 This Open Access Senior Thesis is brought to you by Scholarship@Claremont. It has been accepted for inclusion in this collection by an authorized administrator. For more information, please contact [email protected]. Claremont McKenna College The Mathematical Landscape A guided tour Submitted To Professor Asuman G. Aksoy and Dean Gregory Hess By Antonio Collazo For Senior Thesis Spring 2011 April 25, 2011 Abstract The intent of this paper is to present the reader will enough information to spark a curiosity in to the subject. By no means, is the following a complete formulation of any of the topics covered. I want to give the reader a tour of the mathematical landscape, hoping maybe to see them again. There is plenty of further details to explore in each section, I have just touched the tip the iceberg. The work is basically in four sections: Numbers, Geometry, Functions, Sets and Logic, which are the basic building block of Math. The first sections are a exposition into the mathematical objects and their algebras. The last section dives into the foundation of math, sets and logic, and develops the \language" of Math. My hope is that after this, the read will have the necessarily (maybe not sufficient) information needed to talk the language of Math. Antonio Collazo What is Mathematics? Take a random sample from our population, and ask them \What is Mathematics?" Their answer, most likely, is that Mathematics is about numbers; some will add that Mathematics is the study of numbers and their arithmetic.
    [Show full text]
  • UC Berkeley UC Berkeley Electronic Theses and Dissertations
    UC Berkeley UC Berkeley Electronic Theses and Dissertations Title Propositional Quantification and Comparison in Modal Logic Permalink https://escholarship.org/uc/item/78w732g8 Author DING, YIFENG Publication Date 2021 Peer reviewed|Thesis/dissertation eScholarship.org Powered by the California Digital Library University of California Propositional Quantification and Comparison in Modal Logic by Yifeng Ding A dissertation submitted in partial satisfaction of the requirements for the degree of Doctor of Philosophy in Logic and the Methodology of Science in the Graduate Division of the University of California, Berkeley Committee in charge: Associate Professor Wesley H. Holliday, Chair Professor Shamik Dasgupta Professor Paolo Mancosu Professor Dana S. Scott Professor Seth Yalcin Spring 2021 Propositional Quantification and Comparison in Modal Logic Copyright 2021 by Yifeng Ding 1 Abstract Propositional Quantification and Comparison in Modal Logic by Yifeng Ding Doctor of Philosophy in Logic and the Methodology of Science University of California, Berkeley Associate Professor Wesley H. Holliday, Chair We make the following contributions to modal logics with propositional quantifiers and modal logics with comparative operators in this dissertation: • We define a general notion of normal modal logics with propositional quantifiers. We call them normal Π-logics. Then, as was done by Scrogg's theorem on extensions of the modal logic S5, we study in general the normal Π-logics extending S5. We show that they are all complete with respect to their algebraic semantics based on complete simple monadic algebras. We also show that the lattice formed by these logics is isomorphic to the lattice of the open sets of the disjoint union of two copies of the one-point compactification of N with the natural order topology.
    [Show full text]
  • Solutions 1. Prove That a Binary Relation R Is Transitive Iff R R ⊆ R
    Pencil and Paper Exercises Week 2 — Solutions 1. Prove that a binary relation R is transitive iff R ◦ R ⊆ R. Answer: ⇒: Assume R is a transitive binary relation on A. To be proved: R ◦ R ⊆ R. Proof. Let (x, y) ∈ R ◦ R. We must show that (x, y) ∈ R. From the definition of ◦: ∃z ∈ A :(x, z) ∈ R, (z, y) ∈ R. It follows from this and transitivity of R that (x, y) ∈ R. ⇐: Assume R ◦ R ⊆ R. To be proved: R is transitive. Proof. Let (x, y) ∈ R, (y, z) ∈ R. Then (x, z) ∈ R ◦ R. Since R ◦ R ⊆ R, it follows from this that (x, z) ∈ R. Thus, R is transitive. 2. Give an example of a transitive binary relation R with the property that R◦R 6= R. Answer: The simplest example is a relation consisting of a single pair, say R = {(1, 2)}. This relation is transitive, but R ◦ R = ∅ 6= R. 3. Let R be a binary relation on a set A. Prove that R∪{(x, x) | x ∈ A} is the reflexive closure of R. Answer: Let I = {(x, x) | x ∈ A}. It is clear that R ∪ I is reflexive, and that R ⊆ R ∪ I. To show that R ∪ I is the smallest relation with these two properties, suppose S is reflexive and R ⊆ S. Then by reflexivity of S, I ⊆ S. It follows that R ∪ I ⊆ S. 4. Prove that R ∪ Rˇ is the symmetric closure of R. Answer: Clearly, R ∪ Rˇ is symmetric, and R ⊆ R ∪ Rˇ. Let S be any symmetric relation that includes R.
    [Show full text]
  • You May Not Start to Read the Questions Printed on the Subsequent Pages of This Question Paper Until Instructed That You May Do So by the Invigilator – 2 – PHT0/3
    PHT0/3 PHILOSOPHY TRIPOS Part IA Tuesday 25 May 2004 9 to 12 Paper 3 LOGIC Answer four questions only; at least one from each section. Write the number of the question at the beginning of each answer. Please answer all parts of each numbered question chosen. You may not start to read the questions printed on the subsequent pages of this question paper until instructed that you may do so by the Invigilator – 2 – PHT0/3 SECTION A 1 (a) Explain what is meant by: (i) a symmetric relation (ii) a transitive relation (iii) a reflexive relation (iv) an equivalence relation. (b) Let us say that a relation R is 'Euclidean' iff, for any x and y and z, if Rxy and Rxz then Ryz. (i) Give an example of a Euclidean relation that is neither symmetric nor reflexive. (ii) Show (by an informal argument or otherwise) that any transitive symmetric relation is Euclidean. (iii) Show (by an informal argument or otherwise) that any reflexive Euclidean relation is an equivalence relation. 2 Translate the following sentences into QL= (the language of the predicate calculus with identity), explaining the translation scheme you use. (a) All athletes love Jacques. (b) Some athletes who are philosophers are not logicians. (c) Only an athlete loves a logician. (d) Jacques, the well-known athlete, is not a logician. (e) Whomever Kurt loves admires some logician. (f) All philosophers love Kurt, but some of them also love Jacques. (g) No logician loves everyone loved by Kurt. (h) Only if Kurt is a logician is every student who is a philosopher a logician too.
    [Show full text]
  • Evidence of Evidence in Epistemic Logic
    1 Evidence of Evidence in Epistemic Logic [draft of 24 August 2017; final version to appear in Mattias Skipper Rasmussen and Asbjørn Steglich-Petersen (eds.), Higher-Order Evidence: New Essays, Oxford: Oxford University Press] Timothy Williamson The slogan ‘Evidence of evidence is evidence’ may sound plausible, but what it means is far from clear. It has often been applied to connect evidence in the current situation to evidence in another situation. The relevant link between situations may be diachronic (White 2006: 538): is present evidence of past or future evidence of something present evidence of that thing? Alternatively, the link may be interpersonal (Feldman 2007: 208): is evidence for me of evidence for you of something evidence for me of that thing? Such inter- perspectival links have been discussed because they can destabilize inter-perspectival disagreements. In their own right they have become the topic of a lively recent debate (Fitelson 2012, Feldman 2014, Roche 2014, Tal and Comesaña 2014). This chapter concerns putative intra-perspectival evidential links. Roughly, is present evidence for me of present evidence for me of something present evidence for me of that thing? Unless such a connection holds between a perspective and itself, it is unlikely to hold generally between distinct perspectives. Formally, the single-perspective case is also much simpler to study. Moreover, it concerns issues about the relation between first-order and higher-order evidence, the topic of this volume. The formulations in this chapter have not been tailored for optimal fit with previous discussions. Rather, they are selected because they make an appropriate starting-point, simple, significant, and not too ad hoc.
    [Show full text]
  • Propositional Quantification and Comparison in Modal Logic By
    Propositional Quantification and Comparison in Modal Logic by Yifeng Ding A dissertation submitted in partial satisfaction of the requirements for the degree of Doctor of Philosophy in Logic and the Methodology of Science in the Graduate Division of the University of California, Berkeley Committee in charge: Associate Professor Wesley H. Holliday, Chair Professor Shamik Dasgupta Professor Paolo Mancosu Professor Dana S. Scott Professor Seth Yalcin Spring 2021 Propositional Quantification and Comparison in Modal Logic Copyright 2021 by Yifeng Ding 1 Abstract Propositional Quantification and Comparison in Modal Logic by Yifeng Ding Doctor of Philosophy in Logic and the Methodology of Science University of California, Berkeley Associate Professor Wesley H. Holliday, Chair We make the following contributions to modal logics with propositional quantifiers and modal logics with comparative operators in this dissertation: • We define a general notion of normal modal logics with propositional quantifiers. We call them normal Π-logics. Then, as was done by Scrogg's theorem on extensions of the modal logic S5, we study in general the normal Π-logics extending S5. We show that they are all complete with respect to their algebraic semantics based on complete simple monadic algebras. We also show that the lattice formed by these logics is isomorphic to the lattice of the open sets of the disjoint union of two copies of the one-point compactification of N with the natural order topology. Further, we show how to determine the computability of normal Π-logics extending S5Π. A corollary is that they can be of arbitrarily high Turing-degree. • Regarding the normal Π-logics extending the modal logic KD45, we identify two im- 8 portant axioms: Immod : 8p(p ! p) and 4 : 8p' ! 8p'.
    [Show full text]
  • Typology of Axioms for a Weighted Modal Logic Bénédicte Legastelois, Marie-Jeanne Lesot, Adrien Revault D’Allonnes
    Typology of Axioms for a Weighted Modal Logic Bénédicte Legastelois, Marie-Jeanne Lesot, Adrien Revault d’Allonnes To cite this version: Bénédicte Legastelois, Marie-Jeanne Lesot, Adrien Revault d’Allonnes. Typology of Axioms for a Weighted Modal Logic. International Journal of Approximate Reasoning, Elsevier, 2017, 90, pp.341- 358. 10.1016/j.ijar.2017.06.011. hal-01558038 HAL Id: hal-01558038 https://hal.sorbonne-universite.fr/hal-01558038 Submitted on 29 Sep 2017 HAL is a multi-disciplinary open access L’archive ouverte pluridisciplinaire HAL, est archive for the deposit and dissemination of sci- destinée au dépôt et à la diffusion de documents entific research documents, whether they are pub- scientifiques de niveau recherche, publiés ou non, lished or not. The documents may come from émanant des établissements d’enseignement et de teaching and research institutions in France or recherche français ou étrangers, des laboratoires abroad, or from public or private research centers. publics ou privés. Typology of axioms for a weighted modal logic ∗ a, a b Bénédicte Legastelois , Marie-Jeanne Lesot , Adrien Revault d’Allonnes a Sorbonne Universités, UPMC Univ. Paris 06, CNRS, LIP6 UMR 7606, 4 place Jussieu 75005 Paris, France b Université Paris 8 – EA 4383 – LIASD, FR-93526, Saint-Denis, France a b s t r a c t This paper introduces and studies extensions of modal logics by investigating the soundness of classical modal axioms in a weighted framework. It discusses the notion of relevant weight values, in a specific weighted Kripke semantics and exploits accessibility relation properties. Different generalisations of the classical axioms are constructed and, from these, a typology of weighted axioms is built, distinguishing between four types, Keywords: depending on their relations to their classical counterparts and to the, possibly equivalent, Modal logics frame conditions.
    [Show full text]