Catálogo de publicaciones - libros


Typed Lambda Calculi and Applications: 7th International Conference, TLCA 2005, Nara, Japan, April 21-23, 2005, Proceedings

Paweł Urzyczyn (eds.)

En conferencia: 7º International Conference on Typed Lambda Calculi and Applications (TLCA) . Nara, Japan . April 21, 2005 - April 23, 2005

Resumen/Descripción – provisto por la editorial

No disponible.

Palabras clave – provistas por la editorial

No disponibles.

Disponibilidad
Institución detectada Año de publicación Navegá Descargá Solicitá
No detectada 2005 SpringerLink

Información

Tipo de recurso:

libros

ISBN impreso

978-3-540-25593-2

ISBN electrónico

978-3-540-32014-2

Editor responsable

Springer Nature

País de edición

Reino Unido

Fecha de publicación

Información sobre derechos de publicación

© Springer-Verlag Berlin Heidelberg 2005

Tabla de contenidos

Typed Lambda Calculi and Applications

Paweł Urzyczyn (eds.)

Pp. No disponible

Completeness Theorems and λ-Calculus

Thierry Coquand

The purpose of this note is to present a variation of Hindley’s completeness theorem for simply typed λ -calculus based on Kripke model. This variation was obtained indirectly by simplifying an analysis of a fragment of polymorphic λ -calculus [2].

- Completeness Theorems and -Calculus | Pp. 1-9

A Tutorial Example of the Semantic Approach to Foundational Proof-Carrying Code: Abstract

Amy P. Felty

Proof-carrying code provides a mechanism for insuring that a host, or code consumer, can safely run code delivered by a code producer. The host specifies a safety policy as a set of axioms and inference rules. In addition to a compiled program, the code producer delivers a formal proof of safety expressed in terms of those rules that can be easily checked. Foundational proof-carrying code (FPCC) provides increased security and greater flexibility in the construction of proofs of safety. Proofs of safety are constructed from the smallest possible set of axioms and inference rules. For example, typing rules are not included. In our semantic approach to FPCC, we encode a semantics of types from first principles and the typing rules are proved as lemmas. In addition, we start from a semantic definition of machine instructions and safety is defined directly from this semantics.

- Completeness Theorems and -Calculus | Pp. 10-10

Can Proofs Be Animated By Games?

Susumu Hayashi

Proof animation is a way of executing proofs to find errors in the formalization of proofs. It is intended to be “testing in proof engineering”. Although the realizability interpretation as well as the functional interpretation based on limit-computations were introduced as means for proof animation, they were unrealistic as an architectural basis for actual proof animation tools. We have found game theoretical semantics corresponding to these interpretations, which is likely to be the right architectural basis for proof animation.

- Completeness Theorems and -Calculus | Pp. 11-22

Untyped Algorithmic Equality for Martin-Löf’s Logical Framework with Surjective Pairs

Andreas Abel; Thierry Coquand

An untyped algorithm to test βη -equality for Martin-Löf’s Logical Framework with strong Σ -types is presented and proven complete using a model of partial equivalence relations between untyped terms.

Palabras clave: Type Theory; Logical Framework; Dependent Pair; Conversion Algorithm; Extensionality Rule.

- Contributed Papers | Pp. 23-38

The Monadic Second Order Theory of Trees Given by Arbitrary Level-Two Recursion Schemes Is Decidable

Klaus Aehlig; Jolie G. de Miranda; C. -H. Luke Ong

A tree automaton can simulate the successful runs of a word or tree automaton working on the word or tree denoted by a level-2 lambda-tree. In particular the monadic second order theory of trees given by arbitrary, rather than only by safe, recursion schemes of level 2 is decidable. This solves the level-2 case of an open problem by Knapik, Niwiński and Urzyczyn.

Palabras clave: Order Theory; Variable Node; Recursion Equation; Reduction Sequence; Tree Automaton.

- Contributed Papers | Pp. 39-54

A Feasible Algorithm for Typing in Elementary Affine Logic

Patrick Baillot; Kazushige Terui

We give a new type inference algorithm for typing lambda-terms in Elementary Affine Logic (EAL), which is motivated by applications to complexity and optimal reduction. Following previous references on this topic, the variant of EAL type system we consider (denoted EAL^*) is a variant where sharing is restricted to variables and without polymorphism. Our algorithm improves over the ones already known in that it offers a better complexity bound: if a simple type derivation for the term t is given our algorithm performs EAL^* type inference in polynomial time in the size of the derivation.

- Contributed Papers | Pp. 55-70

Practical Inference for Type-Based Termination in a Polymorphic Setting

Gilles Barthe; Benjamin Grégoire; Fernando Pastawski

We introduce a polymorphic λ -calculus that features inductive types and that enforces termination of recursive definitions through typing. Then, we define a sound and complete type inference algorithm that computes a set of constraints to be satisfied for terms to be typable. In addition, we show that Subject Reduction fails in a naive use of typed-based termination for a λ -calculus à la Church, and we propose a general solution to this problem.

Palabras clave: Constraint System; Inference Algorithm; Typing Rule; Proof Assistant; Inductive Type.

- Contributed Papers | Pp. 71-85

Relational Reasoning in a Nominal Semantics for Storage

Nick Benton; Benjamin Leperchey

We give a monadic semantics in the category of FM-cpos to a higher-order CBV language with recursion and dynamically allocated mutable references that may store both ground data and the addresses of other references, but not functions. This model is adequate, though far from fully abstract. We then develop a relational reasoning principle over the denotational model, and show how it may be used to establish various contextual equivalences involving allocation and encapsulation of store.

Palabras clave: Operational Semantic; Logical Relation; Garbage Collection; Relational Reasoning; Denotational Semantic.

- Contributed Papers | Pp. 86-101

Filters on CoInductive Streams, an Application to Eratosthenes’ Sieve

Yves Bertot

We present the formal description of an algorithm to filter values from an infinite steam using a type theory based prover. The key aspect is that filters are partial co-recursive functions and we solve the problem of expressing partiality. We then show how to prove properties of this filter algorithm and we study an application computing the stream of all prime numbers.

Palabras clave: Prime Number; Type Theory; Recursive Function; Linear Temporal Logic; Recursive Call.

- Contributed Papers | Pp. 102-115