# HG changeset patch # User Christian Urban # Date 1319276590 -3600 # Node ID f329c1f3b36563fed83f8d92d1aa2db3249bed8e # Parent 9e036cad865404023262b7eaebcef46b4dad98b8 initial real diff -r 9e036cad8654 -r f329c1f3b365 index.html --- a/index.html Sat Oct 22 10:37:59 2011 +0100 +++ b/index.html Sat Oct 22 10:43:10 2011 +0100 @@ -1,10 +1,280 @@ - - - - Minimal HTML Document - - - -Test - - + + + +Homepage of Christian Urban + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + +
+ +Links
+Home
+Publications
+Teaching
+Recent Talks
+My Research Group +
+
+ +Handy Information
+People in Logic
+Programming Languages
+Miscellaneous +

+ + + +
+ + + + + + +
+

Christian Urban

+ +E-mail +urbanc at in tum de
+
+ +Address +Institute for Computer Science +at the TU Munich (IV), Boltzmannstrasse 3, D-85748 Garching, Germany. +

+ +Fax +49 89 289 17307 +
+ +
+

+Isabelle Documentation Project (contains now a draft of a 200-page tutorial on Isabelle programming)
+

+Current Position +I have been awarded an +Emmy-Noether +fellowship +to head an independent research group in +the Computer Science Department at the +TU Munich. This group co-operates +with the Theorem Proving Group +chaired by Prof. Tobias Nipkow and +is accommodated by the institute of +Prof. Manfred Broy. +

+ +Past Positions +Between September 2008 and February 2009, I was an invited research fellow in +the Department of Computer Science in Princeton. +In 2004/05 I was an Alexander-von-Humboldt fellow in Munich and +from 2000 until 2004 I was awarded a Research Fellowship in Cambridge. Before that +I did my PhD in Cambridge. +

+ +Research Interests theorem provers, programming languages, compilers, +algorithms, proof theory, type systems, concurrency, lambda calculus, unification, +regular expressions, computability, complexity, functional and logic programming. +

+ +Conferences +UNIF'06 (member of PC), +LFMTP'07 (member of PC), +LFMTP'08 (PC co-chair), +WMM'08 (member of PC), +LSFA'08 (invited speaker), +TAASN'09 (member of PC), +LSFA'09 (member of PC), +IDW'09 (organiser), +WMM'09 (PC chair), +TPHOLs'09 (PC co-chair), +Automatheo'10 (member of PC), +ITP'10 (member of PC), +UNIF'10 (invited speaker), +WMM'10 (invited speaker), +IDW'10 (co-organiser), +CPP'11 (member of PC), +RTA'11 (member of PC), +LFMTP'11 (member of PC) +
+ +

+Nominal Isabelle +I currently work on Nominal +Isabelle. This is joint work with +Dr Stefan Berghofer, +Dr Markus Wenzel, +Dr Cezary Kaliszyk and +the Isabelle-team in Munich. +Many of the theoretical ideas originate from the nominal logic project - a wonderful project headed +by Prof. Andrew Pitts. +The aim of my work is to make formal reasoning involving binders as simple as +on paper and the hope is to lure +masses to automated +theorem proving. My funding for this work was provided in 2004 and 2005 by a research +fellowship from the +Alexander-von-Humboldt +foundation. During this time I was a visitor in the group of +Prof. Helmut Schwichtenberg. +Since 2006 this work is supported by an +Emmy-Noether +fellowship. +There is a webpage and a +mailing list +about Nominal Isabelle. It also includes a list of projects that use Nominal Isabelle. +Users of Nominal Isabelle had their papers appearing at LICS, POPL, FOSSACS, SOS, TPHOLs and CPP. +
+Myhill-Nerode and Regular Expressions +Out of frustration of having to teach inductions in theorem provers using worn-out examples like +fib and even/odd, we implemented a large part of regular language theory in Isabelle/HOL. +This implementation +gives rise to much more interesting examples, as shown +here and +here. It turns out that +formalisations of automata theory are a huge +pain +in theorem provers, especially in those that are HOL-based. +We therefore went against the +mainstream +and used in our formalisation regular expressions exclusively, +because they are much more convenient for formal reasoning. The results we +formalised include: the Myhill-Nerode theorem, the closure of regular languages +under complementation, finiteness of derivatives of regular expressions and a surprising +result about Subseq, which according to +this +blog +should be better known. This is joint work with Prof. Xingyuan +Zhang and his student Chunhan Wu from the +PLA University of Science and Technology in Nanjing. +My funding for this work came from the +Chinese-German Research Centre. +
+Nominal Unification and Alpha-Prolog +Nominal unification is one outcome of +my involvement in the nominal logic project in Cambridge. Another is the logic programming language +alpha-Prolog (joint work with Dr James Cheney), +which uses nominal unification - click for details +here. +The nominal unification algorithm has been +formally verified in Isabelle. This +was possible since this unification algorithm is formulated in a simple first-order language +(unlike other algorithms for higher-order unification). +Prof. Daniel Friedman and his group use nominal +unification in their alpha-Kanren system implemented in Scheme. +Prof. Maribel Fernandez and her student +improved the nominal unification algorithm to be quadratic. +My funding for this work was provided through a research fellowship from +Corpus Christi College, Cambridge. +
+Classical Logic +I was Ph.D. student in the University of Cambridge +Computer Laboratory +and for three years +called Gonville and Caius College my home. I was very lucky to have +Dr Gavin Bierman +as supervisor. My research in Cambridge was also very much influenced by +Prof. Martin Hyland. +Some details on my thesis "Classical Logic and Computation" are +elsewhere, including +a Java Applet that +'visualises' some of the results from the thesis. I completed the writing of +the thesis in Marseille in the group of +Prof. Jean-Yves Girard. My study in +Cambridge was funded by two scholarships +from the German government; my year in Marseille by a TMR-fellowship from the EU. +My PhD was also one starting point for the EPSRC Project on the Semantics of Classical +Proofs. The strong normalisation result in the PhD has recently been used by +Prof. Claude Kirchner and his +students to prove consistency for their superdeduction system lemuridae. +
+Forum +I implemented Forum, a programming language based on classical linear logic, +as my M.Phil. thesis. This was joint work with +Dr Roy Dyckhoff. +Details can be found +here and +here. During my +M.Phil study I spent one month in Philadelphia invited by +Prof. Dale Miller. +
+G4ip An implementation of G4ip using the imperative language Pizza can be found +here. +Pizza is a conservative +extension of Java and a precursor of Scala. The implementation illustrates the technique of success +continuations. +
+

+ +Last modified: Mon Sep 5 10:11:36 BST 2011 + +[Validate this page.] + + + + diff -r 9e036cad8654 -r f329c1f3b365 logic.html --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/logic.html Sat Oct 22 10:43:10 2011 +0100 @@ -0,0 +1,158 @@ + + + +Homepage of Christian Urban + + + + + + + + + + + + + + + + +
+ +Links
+Home
+Publications
+Teaching
+Recent Talks
+My Research Group +
+
+ +Handy Information
+People in Logic
+Programming Languages
+Miscellaneous +

+ + + + + +
+

Logic Related Links

+ +

An Incomplete List of People Working in Logic, Proof Theory, Theorem Provers and Related Areas

+ + + + + + + +
+
+ +
Andrew Appel
+
Andrew Pitts
+
Amy Felty
+
Benjamin Pierce
+
Catuscia Palamidessi
+
Claudia Faggian
+
Dale Miller
+
Daniel Friedman
+
David Pym
+
Didier Galmiche
+
Edmund Robinson
+
Frank Pfenning
+
Gavin Bierman
+
George Necula
+
Gianluigi Bellin
+
Gilles Dowek
+
Glynn Winskel
+
Gopalan Nadathur
+
Gordon Plotkin
+
Helmut Schwichtenberg
+
Henk Barendregt
+
Hugo Herbelin
+
Iliano Cervesato +
James Cheney +
Jean Gallier, + papers
+
Jean-Yves Girard
+
John Harrison
+
John Mitchell
+
Karl Crary
+
+
+
+
Larry Paulson
+
Luke Ong
+
Martin Hofmann
+
Martin Hyland
+
Markus Wenzel
+
Matthias Baaz
+
Matthias Felleisen
+
Michael Norrish
+
Mitchell Wand
+
Neil Jones
+
Nick Benton
+
Peter Homeier +
Peter Sewell +
Phil Scott
+
Philip Wadler
+
Pierre-Louis Curien
+
Randy Pollack
+
René Vestergaard
+
Robert Constable
+
Robert Harper
+
Roy Dyckhoff
+
Samson Abramsky
+
Steffen Hölldobler
+
Solomon Feferman
+
Stefan Berghofer
+
Steve Zdancewic
+
Thierry Coquand
+
Tobias Nipkow
+
Ulrich Berger
+
Xavier Leroy
+
+
+ +

Bookmarks

+ +
+
+ Pi-calculus
+
+ Survey on linear logic programming languages by Dale Miller
+
+ Researchers in Rewriting
+
+ List of open problems in term rewriting
+
+ Mathematical logic
+
Computability Logic Homepage +
+ + +
+

+ +Last modified: Mon Mar 29 08:15:12 CEST 2010 + +[Validate this page.] + + diff -r 9e036cad8654 -r f329c1f3b365 misc.html --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/misc.html Sat Oct 22 10:43:10 2011 +0100 @@ -0,0 +1,117 @@ + + + + Christian Urban + + + + + + + + + + + + + + + + + + + + + +
+ +Links
+Home
+Publications
+Teaching
+Recent Talks
+My Research Group +
+
+ +Handy Information
+People in Logic
+Programming Languages
+Miscellaneous +

+ + + + +
+

GNU/Linux World

+
+ Linux Documentation Project +
+ Xemacs +
+ XOrg + (Mailing Lists) +
+ CTAN Catalogue +
+ TeX Live +
+ TeX Users Group + (Mailing Lists) +
+ Slashdot +
+ Linux Weekly News +
+ Linux-Kernel Archive + (Mailing List) +
+ Slackware, + + Slackware-Ftp, + + Packages, + + Forum +
+ KDE Desktop + (Mailing Lists) +
+ The Risks Digest +
+ C. of ACM Inside Risks +
+ Beamer Latex Class +
+
+

Airlines and Railways

+
+ British Airways, + Lufthansa, + Deutsche Bundesbahn, + Ryanair, + Easyjet, + World Times +
+
+

+ +Last modified: Mon Feb 16 23:17:30 GMT 2009 + +[Validate this page.] + + diff -r 9e036cad8654 -r f329c1f3b365 new.gif Binary file new.gif has changed diff -r 9e036cad8654 -r f329c1f3b365 picture-small.jpg Binary file picture-small.jpg has changed diff -r 9e036cad8654 -r f329c1f3b365 picture.jpg Binary file picture.jpg has changed diff -r 9e036cad8654 -r f329c1f3b365 publications.html --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/publications.html Sat Oct 22 10:43:10 2011 +0100 @@ -0,0 +1,426 @@ + + + + Christian Urban + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + +
+ +Links
+Home
+Publications
+Teaching
+Recent Talks
+My Research Group +
+
+ +Handy Information
+People in Logic
+Programming Languages
+Miscellaneous +

+ + + + +
+

Publications

+Warning: +Currently not all papers are available from this page. +Please email me for copies of the papers you cannot find. +
+

Pending

+ +

Mechanizing the Metatheory of Mini-XQuery. + (with Cheney) To appear at CPP 2011. + [pdf] + +

A Formalisation of the Myhill-Nerode Theorem based on Regular Expressions. + (with Wu and Zhang) Journal version. Submitted. + [pdf] + +

General Bindings and Alpha-Equivalence in Nominal Isabelle. + (with Kaliszyk) Journal version. Submitted. + [pdf] + +

How to Prove False using the Variable Convention. + Appears as a poster at TTVSI, 1 page. + [pdf] + [poster] + +

Strong Induction Principles in the Locally Nameless + Representation of Binders (Preliminary Notes). (with Pollack) A shorter version + of this paper was accepted at WMM'07. + [pdf] +

+

2011

+

General Bindings and Alpha-Equivalence in Nominal Isabelle. + (with Kaliszyk) + In Proceedings of the 20th European Symposium on Programming (ESOP 2011). + In Volume 6602 of Lecture Notes in Computer Science. Pages 480-500. + © Springer Verlag + [pdf] + +

A Formalisation of the Myhill-Nerode Theorem based on Regular Expressions (Proof + Pearl). + (with Wu and Zhang) + In Proceedings of the 2nd Conference on Interactive Theorem Proving (ITP 2011). + In Volume 6898 of Lecture Notes in Computer Science. Pages 341-356. + © Springer Verlag + [pdf] + +

Quotients Revisited for Isabelle/HOL. + (with Kaliszyk) In Proceedings of the ACM Symposium on Applied + Computing (SAC 2011), Software Verification and Testing track, + Pages 1639-1644. + [pdf] +

+

2010

+

Proof Pearl: A New Foundation for Nominal Isabelle. (with Huffman) + In Proceedings of the 1st Conference on Interactive Theorem Proving (ITP 2010). + In Volume 6172 of Lecture Notes in Computer Science. Pages 35-50. + © Springer Verlag + [pdf] + +

Mechanizing the Metatheory of LF. (with Cheney and Berghofer) + In + ACM Transactions on Computational Logic, Vol 12(2), Pages 15:1 - 15:42, 2011. + [technical report] + +

Nominal Unification Revisited. + (invited paper) In Proceedings of the 24th Workshop on Unification (UNIF 2010). + In Volume 42 of Electronic Proceedings in Theoretical Computer Science. Pages 1-11, 2010. + [pdf] + +

+

2009

+

Nominal Formalisations of Typical SOS Proofs. + (with Narboux) In Proceedings of the 3rd Workshop on Logical and Semantic + Frameworks with Applications (LFSA'08). Electronic + Notes in Theoretical Computer Science, 247, Pages 139-155, 2009. + [pdf]. + +

Proceedings of Theorem Proving in Higher Order Logics (TPHOLs'09). + (with Berghofer, Nipkow and Wenzel) Volume 5674 of Lecture Notes in + Computer Science, 2009. + © Springer Verlag + +

Nominal Verification of W. (with Nipkow) + From Semantics to Computer Science, Essays in Honour of Gilles Kahn, + edited by Bertot, Huet, Levy and Plotkin. Cambridge + University Press, 2009. Pages 363-382. + [pdf] +

+

2008

+

Mechanizing the Metatheory of LF. (with Cheney and Berghofer) In Proceedings of the + 23rd IEEE Symposium on Logic in Computer Science (LICS 2008), IEEE Computer Society, + June 2008. Pages 45-56. + [pdf] More + information is elsewhere. + +

Nominal Inversion Principles. (with Berghofer) + In Proceedings of 21st International Conference on Theorem Proving in + Higher Order Logics (TPHOLs'08). In Volume 5170 of Lecture Notes in + Computer Science. Pages 71-85. + © Springer Verlag + [pdf]

+ + (Note that the proof in figure 3 is chosen as an illustrative example to + show how to use inversion principles (the main topic of the paper). If one + does the induction on the beta-reduction relation, instead of the typing + relation, then the proof is almost trivial and can be found automatically + by Isabelle only using some very standard inversion principles for the + typing relation.) + +

Mechanising a Proof of Craig's Interpolation Theorem for Intuitionistic Logic in + Nominal Isabelle. (with Chapman and McKinna) + In Proceedings of 9th International Conference on Artificial Intelligence + and Symbolic Computation (AISC'08). In Volume 5144 of Lecture Notes in + Artificial Intelligene. Pages 38-52. + © Springer Verlag + + + +

Revisiting Cut-Elimination: One Difficult Proof is Really a Proof. (with Zhu) + In Proceedings of the 19th International Conference on Rewriting Techniques + and Applications (RTA 2008). In Volume 5117 of Lecture Notes in Computer Science. + Pages 409-424. + © Springer Verlag + [pdf]

+ + (This paper corrects some lemmas in my PhD-thesis. The errors were found by formalising + the proof in Nominal Isabelle.) +

+

2007

+

Barendregt's Variable Convention in Rule Inductions. + (with Berghofer and Norrish) In Proceedings of the 21th + Conference on Automated Deduction (CADE 2007). In volume 4603 + of Lecture Notes in Artificial Intelligence. Bremen, Germany. + July 2007. Pages 35-50. + © Springer Verlag + [ps] + +

This paper supersedes the MERLIN-paper from 2005. + +

Nominal Techniques in Isabelle/HOL. In + Journal of Automatic Reasoning, 2008, Vol. 40(4), 327-356. + [ps] + [pdf] + +

Formalising in Nominal Isabelle Crary's Completeness Proof for Equivalence Checking. + (with Narboux) In Proceedings of the International Workshop on Logical Frameworks and + Meta-Languages: Theory and Practice (LFMTP 2007). Electronic Notes in + Theoretical Computer Science. Vol. 196. Pages 3-18. + [pdf]

+ + (There is a minor problem in the statement on page 4 where we write that alpha-renamings + are required in order to show the equivalence of Q-Beta and Q-Beta': While the equivalence + can be proved using alpha-renamings, it can also be proved by a careful analysis of the + available freshness-constraints.) + +

Nominal Logic Programming. (with Cheney) + In + ACM Transactions on Programming Languages and Systems, + 2008, Vol. 30(5), Article 26, pages 1-47. +

+

2006

+

Proof Theory of Classical Propositional Calculus. + (with Hyland, Bellin and Robinson) In Theoretical Computer + Science 2006. Vol. 364(2). Pages 143-170. + [ps] + +

A Recursion Combinator for Nominal Datatypes + Implemented in Isabelle/HOL. (with Berghofer) In Proceedings of the 3rd + International Joint Conference on Automated Deduction (IJCAR 2006). + Seattle, USA. In volume 4130 of Lecture Notes in Artificial Intelligence. + Pages 498-512. + © Springer Verlag + [ps] + +

Classical Logic is better than Intuitionistic Logic: + A Conjecture about Double-Negation Translations. (with Ratiu) In Proceedings + of the 1st International Workshop on Classical Logic and Computation (CL & C 2006). + Venice, Italy. 20pp. + [ps] + +

A Head-to-Head Comparison of de Bruijn Indices and Names. (with Berghofer) + In Proceedings of the International Workshop on Logical Frameworks and + Meta-Languages: Theory and Practice (LFMTP 2006). Electronic Notes in + Theoretical Computer Science. Vol. 174(5). Pages 53-67. + [ps] +

+

2005

+

A Formal Treatment of the Barendregt Variable Convention in Rule Inductions. (with Norrish) + In Proceedings of the ACM Workshop on Mechanized Reasoning about Languages with Variable + Binding and Names (MERLIN 2005). Tallinn, Estonia. September 2005. Pages 25-32. © ACM, Inc. + [ps] + [pdf] +

+ (There was a small typo in the definition of permutation equality, which has been corrected + in the versions above. This paper received favourable comments on the + FOM mailing-list.) + +

Nominal Techniques in Isabelle/HOL. (with Tasson) In Proceedings of the 20th + Conference on Automated Deduction (CADE 2005). In volume 3632 of Lecture Notes in Artificial + Intelligence. Tallinn, Estonia. July 2005. Pages 38-53. + © Springer Verlag + [ps] + +

Avoiding Equivariance in Alpha-Prolog. (with Cheney) In Proceedings of the 7th + International Conference on Typed Lambda Calculi and Applications (TLCA 2005). + In Volume 3461 of Lecture Notes in Computer Science. Nara, Japan. April 2005. Pages 401-416. + © Springer Verlag + [ps] +

+

2004

+

Nominal Unification. (with Pitts and Gabbay) In Theoretical Computer Science + 2004. Vol. 323(1-3). Pages 473-497. + [ps] + [pdf] + +

Nominal Techniques for Reasoning about Formal Languages. Reader for an advanced + course at the ESSLLI summer school. 26 Pages. Appeared as LORIA technical report. + +

Alpha-Prolog: A Logic Programming Language with Names, Binding and Alpha-Equivalence. + (with Cheney) In Proceedings of the International Conference on Logic Programming + (ICLP 2004). In Volume 3132 of Lecture Notes in Computer Science. St-Malo, France. + September 2004. Pages 269-283. + © Springer Verlag + [ps] +

+

2003

+

Nominal Unification. (with Pitts and Gabbay) + In Proceedings of the Computer Science Logic and 8th Kurt Gödel Colloquium + (CSL & KGC 2003). In Volume 2803 of Lecture Notes in Computer Science. Vienna, Austria. + August 2003. Pages 513-527. + © Springer Verlag + [ps] + +

System Description: Alpha-Prolog, a Fresh Approach to Logic Programming Modulo + Alpha-Equivalence. (with Cheney) In Proceedings of the 17th International Workshop on + Unification, UNIF'03. Valencia, Spain. June 2003. Technical Report + DSIC-II/12/03, Departamento de Sistemas Informaticos y Computacion, + Universidad Politecnica de Valencia, 2003. Pages 15-19. + [ps] + +

Work in Progress: Logic Programming with Names and Binding. (with Cheney) + CoLogNet Newsletter No. 4, 2003. Pages 25-28. + [ps] +

+

2002

+

Strong Normalisation of Herbelin's Explicit Substitution Calculus with + Substitution Propagation. + (with Dyckhoff) Journal of Logic and Computation, Volume 13, No 5, Pages 689-706. + [pdf] + + +

+

2001

+

Strong Normalisation of Cut-Elimination in Classical Logic. (with Bierman) + Fundamenta Informaticae, 45(1-2), January 2001, Pages 123-155. + [ps.gz] + [pdf] + +

Strong Normalisation of Herbelin's Explicit Substitution Calculus with + Substitution Propagation. (with Dyckhoff) In Proceedings of the 4th + Workshop on Explicit Substitutions Theory and Applications (WESTAPP'01). + Logic Group Preprint series No 210. Utrecht, the Netherlands. May 2001. Pages 26-45. + [pdf] + +

Strong Normalisation for a Gentzen-like Cut-Elimination Procedure. + In Proceedings of the 5th International Conference on Typed Lambda Calculi and + Applications (TLCA 2001). In Volume 2044 of Lecture Notes in + Computer Science. Krakow, Poland. May 2001. Pages 415-429. + © Springer Verlag + [ps.gz] + [pdf] +

+

2000

+

Classical Logic and Computation. +Ph.D. Thesis, University of Cambridge. Supervised by Dr Gavin Bierman. October 2000. +Some details are elsewhere. +[ps.gz] +

+

1999

+

Strong Normalisation of Cut-Elimination in Classical Logic. +(with Bierman) In Proceedings of the 5th International Conference on Typed +Lambda Calculi and Applications (TLCA 1999). In Volume 1581 of Lecture Notes in +Computer Science. L'Aquila, Italy. April 1999. Pages 365-380. +© Springer Verlag +[ps.gz] +[pdf] +

+

1998

+

Implementation of Proof Search in the Imperative Programming Language Pizza. +In Proceedings of the 7th International Conference on Automated Reasoning with +Analytic Tableaux and Related Methods (TABELAUX 1998). In Volume 1397 of Lecture Notes in +Artificial Intelligence. Oisterwijk, the Netherlands. May 1998. Pages 313-319. +© Springer Verlag +[ps.gz] +

+

1996

+

Forum and Its Implementation. +M.Phil. Thesis, University of St Andrews. Supervised by Dr Roy Dyckhoff. April 1996. +

+

+ +Last modified: Tue Sep 20 16:01:02 CEST 2011 + +[Validate this page.] + + diff -r 9e036cad8654 -r f329c1f3b365 teaching.html --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/teaching.html Sat Oct 22 10:43:10 2011 +0100 @@ -0,0 +1,356 @@ + + + + Christian Urban + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + + +
+ +Links
+Home
+Publications
+Teaching
+Recent Talks
+My Research Group +
+
+ +Handy Information
+People in Logic
+Programming Languages
+Miscellaneous +

+ + + + +
+

Teaching

+ +

Undergraduate students who have written dissertations under my supervision: +

    +
  • Dominik Wee (2002-2003, King's College, Cambride; now at McKinsey in Munich) +Part-II dissertation: An Implementation of Alpha-Prolog, +A Logic Programming Language with Support for Binding Syntax (out of 84 dissertations, Dominik's +thesis received the Data Connection prize for the highest number of marks awarded in 2003)
  • +
  • Lisa White (2003-2004, Corpus, Cambridge) Part-II dissertation: Hal 2004, A Nominal Theorem +Prover
  • +
  • Christine Tasson +(2004, ENS Cachan, France; now in the PPS group in Paris) +Induction Principles for Alpha-Equated Lambda-Terms +(the paper coming out of this work was presented at CADE)
  • +
  • Mathilde Arnaud +(2007, ENS Cachan, France) Formalization of Generative Unbinding
  • +
+ + +
+ +

2010-2011

+ +

Spring +

    +
  • one-day tutorial on Nominal Isabelle at POPL'11 with Cezary Kaliszyk +
+ +

Autumn +

    +
  • Types course at the University of Cambridge (Mondays, +Wednesdays and Fridays at 10 o'clock in Lecture Theater 2, starting 8th October) +[Lec 1] +[Lec 2] +[Lec 3] +[Lec 4] +[Lec 5] +[Lec 6] +[Lec 7] +[Lec 8] +
  • two-day Isabelle/Isar tutorial at the University Paris Sud with Markus Wenzel +
+
+

2009-2010

+ +

Summer +

+
+

2008-2009

+ +

Summer +

    +
  • a course + on Isabelle at the Chinese Academy of Science (7.5 h) +
  • Pearls in Computer Science, a course for gifted undergraduate students in Munich (5h) +
+ +

Autumn +

+ +
+

2007-2008

+ +

Sommersemester +

+ +
+

2006-2007

+

Wintersemester +

+ + +

Sommersemester +

  • A course at the International School on Rewriting (1.5h)
+
+

2005-2006

+

Wintersemester +

  • Scheme course at the LMU (4h)
  • +
  • a course on nominal datatypes at the University of Pennsylvania + (6.5h, slides of + [Lec 1] + [Lec 2] + [Lec 3] + [Lec 4])
  • +
  • Theory-Minicourse on nominal datatypes in Cambridge + (4h, slides of + [Lec 1] + [Lec 2] + [Lec 3] + [Lec 4])
  • +
  • Club2-course on the nominal datatype package at the TU Munich + (5h, slides of + [Lec 1] + [Lec 2] + [Lec 3] + [Lec 4] + [Lec 5])
  • +
+
+

2004-2005

+

Wintersemester +

Scheme course at the LMU (10h) +
Linear Algebra for Computer Scientists at the LMU (14h) +
Discrete Structures for Computer Scientists at the LMU (12h) +
+

Sommersemester +

A course on my nominal work at the LMU (10h) + (slides of + [Lec 1] + [Lec 2] + [Lec 3] + [Lec 4] + [Lec 5] + [Lec 6] + [Lec 7] + [Lec 8] + [Lec 9] + [Lec 10]) +
+
+

2003-2004

+

Michelmas +

Logic and Proof (4h) +
Discrete Mathematics I (9h) +
Part II project on a Nominal Theorem Assistant (5.5h) +
Interviews of new students (13.5h) +
+

Lent +

Computation Theory (3h) +
Discrete Mathematics II (8h) +
Semantics of Programming Languages (3h) +
Part II project on a Nominal Theorem Assistant (9.5h) +
+

Easter +

Regular Languages and Finite Automata (6h) +
Foundations of Functional Programming (3h) +
Complexity Theory +
+ +

Summer +

Avanced course on nominal logic at the + ESSLLI summerschool in Nancy
+ (slides of + [Day 1] + [Day 2] + [Day 3] + [Day 4] + [Day 5]) +
student intern from the ENS Cachan +
+
+

2002-2003

+

Michelmas +

Logic and Proof (5h) +
Discrete Mathematics I (7h) +
Part II project on Nominal Unification (7h) +
Interviews of new students +
+

Lent +

Computation Theory (5.5h) +
Discrete Mathematics II (8.5h) +
Part II project (5h) +
+

Easter +

Semantics of Programming Languages (4h) +
Regular Languages and Finite Automata (3h) +
Part II project (3.5h) +
+
+

2001-2002

+

Michelmas +

Logic, Computability and Set Theory (for Math students) +
Data Structures and Algorithms +
Logic and Proof (4h) +
Discrete Mathematics I +
Interviews of new students +
+

Lent +

Discrete Mathematics II +
Semantics of Programming Languages +
Computation Theory +
Probablility +
+

Easter +

Regular Languages and Finite Automata +
Complexity Theory +
+
+

previous

+
+
Types +
Denotational Semantics +
Communicating Atomata and Pi-calculus +
Semantics of Programming Languages +
Foundations of Functional Programming +
Probability +
Computation Theory +
Complexity Theory +
Logic, Computation and Set Theory +
+
+

+ +Last modified: Tue Sep 20 15:55:36 CEST 2011 + +[Validate this page.] + + diff -r 9e036cad8654 -r f329c1f3b365 travelling.html --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/travelling.html Sat Oct 22 10:43:10 2011 +0100 @@ -0,0 +1,333 @@ + + + + Christian Urban + + + + + + + + + + + + + + + + + + + + + +
+ +Links
+Home
+Publications
+Teaching
+Recent Talks
+My Research Group +
+
+ +Handy Information
+People in Logic
+Programming Languages
+Miscellaneous +

+ + + + +
+

Talks and Travel Plans

+
    +
  • Talk at ITU, Copenhagen (15 August, host: Prof. Lars Birkedal) +
  • Talk at ITP'11 (22 - 25 August, Nijmegen) +
+
+

Old

+ +
2011
+ +
    +
  • Talk at Tsinghua (28 April - 8 May, host: Prof. Jean-Pierre Jouannaud) +
  • Talk at ECNU, Shanghai (8 - 28 April, host: Prof. Jifeng He) +
  • Talk at ESOP'11 (26 - 30 March, Saarbrücken) +
  • Talk at Uppsala University (3 March, host: Prof. Joachim Parrow) +
  • One-day tutorial + on Nominal Isabelle at POPL 2011 + (21 January, Austin) +
+ + +
2010
+
    +
  • Isabelle/Isar tutorial at University Paris Sud (22 - 23 November, host: Dr Markus Wenzel) +
  • Talk about regular expressions and Myhill-Nerode in Cambridge (9 November) +
  • Talk at the University of Sussex (3 November, host: Dr Martin Berger) +
  • Invited Talk at WMM'10 (25 September) +
  • Talk at the Jiao Tong University (20 September, host: Prof. Kenny Zhu) +
  • Course on Isabelle Programming at the University of Nanjing + (host: Prof. Xingyuan Zhang, 1st - 31st August) +
  • Talk at ITP (Edinburgh, 11 - 14 July) +
  • Invited Talk at UNIF'10 (14 July) +
  • Larry Paulson and Christian organise the Isabelle Developers Workshop (Cambridge, 17 and 18 June) +
  • Talk in the Automated Reasoning Group in Cambridge (8 June) +
  • On the thesis committee of Clement Houtmann (Nancy, 12 March) +
  • Talk in the Automated Reasoning Group in Cambridge (16 February) +
  • POPL (20th - 22nd January) +
+ +
2009
+
    +
  • Schloss Dagstuhl Seminar (4th - 9th October) +
  • visit to Dr James Cheney and ICFP & WMM (Edinburgh, 26th August - 5th September) +
  • Talk at Tsinghua University (22 May, host: Prof. Jean-Pierre Jouannaud) +
  • Isabelle course at the Chinese Academy of Sciences in Beijing (May/June, hosts: Prof. Huimin Lin + and Prof. Yongjian Li) +
  • Talk at Darmstadt (21 April, host: Prof. Helmut Veith) +
  • TAASN (PC member, 22 March, York) +
  • POPL (18th - 24th January) +
+ + +
2008
+
    +
  • Research visit to Princeton University (15th September - 13th December, host: Prof. Andrew Appel) +
  • Talk + at MIT (21th November, hosts Prof. Martin Rinard and Dr Cameron Freer) +
  • Talk at NYU (10th November, host Prof. Benjamin Goldberg) +
  • Kick-off meeting of the + PUMA Doctoral Programme + (28 September - 3 October, Spitzingsee) +
  • Invited Talk at LSFA (26th August, Salvador, Brazil) +
  • Talk (with Berghofer) at TPHOLs (18 - 21 August, Montreal, Canada) +
  • Nominal Isabelle + at IJCAR'08 tutorial + (11 August, Sydney) +
  • A course on Nominal Isabelle at the +Oregon Summer School +on Logic and Theorem Proving in Programming Languages (22 - 30 July, Eugene, 4h, + [Slides 1], + [Slides 2], + [Slides 3], + [Video 1], + [Video 2], + [Video 3]) +
  • Talk at RTA (15 - 17 July, Hagenberg, Austria) +
  • Talk at LICS (24 - 27 June, Pittsburgh) +
  • Talk in Swansea (1 April, hosts: Prof. Roger Hindley, Dr Ulrich Berger) +
  • Poster at TTVSI (25 - 26 March, London) +
  • Talk at the CANS meeting (10 March, King's College London) +
  • Talk at Imperial College London (6 March, host: Dr Philippa Gardner) +
  • Talk at Yale University (24 January, New Haven, host: Prof. Zhong Shao) +
  • Talk at Northeastern University (22 January, Boston, host: Prof. Mitchell Wand) +
  • Invited Researcher at the Indiana University (January, Bloomington, host: Prof. Daniel Friedman) +
  • POPL (7 - 12 January, San Francisco) +
+ +
2007
+
    +
  • Talks at the Saarbrücken University (13 - 14 December, host: Prof. Gerd Smolka) +
  • Thesis examination of Dragisa Zunic (21. December, Lyon) +
  • Talk at Workshop on Mechanizing Metatheory (Freiburg, 1 - 4 October) +
  • TPHOLs (Kaiserslautern, 10 - 13 September) +
  • Talks at CADE and LFMTP in Bremen (15 - 20 July) +
  • Lecture course at the International School on Rewriting in Nancy (2 - 6 July) +
  • Talk at LFCS in Edinburgh (29th May, host: Randy Pollack) +
  • Talk at ICMS Workshop on Substitution and Naming in Computer Science + (26 - 28 May, Edinburgh) +
  • Invited Researcher at the NICTA Institute in Canberra (5 - 24 May, host: Dr Michael Norrish) +
  • Talk at St Andrews University (13th February, host: Dr Roy Dyckhoff) +
  • CANS-workshop (19th March, London) +
+ +
2006
+
    +
  • Talk at the CANS-workshop (26th October, host: Prof. Andrew Pitts) +
  • Talk in London (1st November, host: Prof. Edmund Robinson) +
  • Talk in Amsterdam (15th Setptember, hosts: Prof. Jan Klop and Dr Femke van Raamsdonk) +
  • visit to Prof. Henk Barendregt in Nijmegen (26th September) +
  • Talk at IJCAR-Conference (16 - 21 August, Seattle) +
  • Talk at LFMTP workshop (15th August, Seattle) +
  • Meeting of all Emmy-Noether Fellows (21 - 24 July, Potsdam) +
  • Talk at the CL&C Workshop (15 July, Venice) +
  • Talk at the University of Frankfurt (22 June, host: Prof. Schmidt-Schauss) +
  • Nominal-Sets Meeting in Cambridge (26 April) +
  • Talk at the Types Workshop in Nottingham (18 - 21 April) +
  • Winterhütte vom Lehrstuhl Broy (27 - 29 March) +
  • Talk at PoplMark-Workshop (Charleston, South Carolina, 13 - 16 January) +
+ +
2005
+
    +
  • Talk in Edinburgh (25 January, host: Ian Stark) +
  • Talk in Leicester (28 January, host: Neil Ghani) +
  • Talk at King's College London (2 February, host: Maribel Fernandez) +
  • Talk at RISC in Linz (3 March, host: Bruno Buchberger) +
  • Talk at PPS in Paris (8 March, host: Pierre-Louis Curien) +
  • Oberwolfach workshop on Proof Theory, Type Theory and Constructive Mathematics + (Germany, 20-26 March 2005) +
  • Talk at Arbeitstagung Venedig (28 March - 2 April) +
  • Talk at TLCA'05 in Nara (Japan, 21-23 April) +
  • Talk at JAIST about Binding (Japan, 24 - 25 April, host: Rene Vestergaard) +
  • Talk in Vienna on Cut-Elimination (4 - 6 July, host: Matthias Baaz) +
  • Talk at CADE-20 in Tallinn (24 - 27 July) +
  • Talk at MERLIN-3 in Tallinn (30 September) +
  • Talk at Carnegie Mellon University (11 November, host: Frank Pfenning) +
  • Course at University of Pennsylvania (9 - 21 November, hosts: Benjamin Pierce and Steve Zdancewic) +
  • Course in Cambridge (5 - 8 December) +
  • Talk at the Workshop on Computational Applications of + Nominal Sets in London (CANS, 6 December, hosts: Andrew Pitts and Maribel Fernandez) +
+ +
2004
+
    +
  • Talk on Binding in Isabelle/HOL (Nijmegen, The Netherlands, 1 - 2 November, host: Henk Barendregt) +
  • visit to Prof. Dale Miller in Paris (France, 28 September) +
  • Talk (with Jeney) at ICLP in St Malo (France, 5 - 10 September) +
  • SOS workshop in London (30 August) +
  • Course at ESSLLI 2004 - The 16th European Summer School in + Logic, Language and Information + Advanced Course on Nominal Reasoning (Nancy, France, 9-20 August) +
    + Slides of + [Day 1] + [Day 2] + [Day 3] + [Day 4] + [Day 5] +
  • visit to Dr Claudia Faggian in Padova (Italy, 24 March) +
+
2003
+
    +
  • Talk in Oxford (24 November, host: Luke Ong) +
  • Talk in the theory seminar at the University of Kent (13 October, host: Stefan Kahrs) +
  • Talk at CSL & KGC 2003 Colloquium (Vienna, Austria, 22 - 30 August) +
  • Talk (with Cheney) at UNIF 2003 workshop (Valencia, Spain, 7-13 June) +
  • Talk at the festive TeReSe-Bookday + (Amsterdam, the Netherlands, 3 - 6 June, host: Jan Willem Klop, slides + [ps] + [pdf]) +
  • Talk in Nijmegen (the Netherlands, 14 April, host: Henk Barendregt) +
  • Talk in St Andrews (1 April, host: Roy Dyckhoff) +
  • Talk at Workshop on Proof Theory and Algorithms (Edinburgh, 23 - 29 March) +
  • Talk at LMU (Munich, 20 January, host: Helmut Schwichtenberg) +
+
2002
+ +
2001
+
    +
  • Linear Meeting in Bertinoro, Italy (22 - 25 April) +
  • Talk at the TLCA 2001 + (Krakow, 2 - 5 May) +
  • Talk at the Natural Deduction meeting in Rio de Janeiro (30 June - 7 July, + slides [ps.gz]) +
  • Summer School +Marktoberdorf +(24 July - 5 August) +
+ +
2000
+ + +
1999
+ + +
1998
+
    +
  • Talk at the + Linear Logic and Typed Lambda-Calculus Workshop in Marseille (6 - 10 April) +
  • Talk at the TABLEAUX'98 Conference in Tilburg, the Netherlands (5 - 8 May) +
  • Mathfit Workshop on Concurrency in London (9 - 11 June) +
  • Talk in the Theory Seminar in St Andrews (July, host: Roy Dyckhoff) +
  • Talk at the Linear Meeting in Tende, France (8 - 11 September) +
  • Talk at the AI Dep. in Dresden + (September) +
+ +
1997
+ + +
1996
+
    +
  • ELP'96 in Leipzig (Germany, 28 - 30 March) +
  • BCTCS 12 in Canterbury (1 - 4 April) +
  • Research visit to the UPenn (Philadelphia, 9 May - 3 June) +
  • Meeting with + Dr Gavin Bierman and + Dr Martin Hyland in Cambridge (6 - 7 June) +
  • KI'96 in Dresden (17 - 19 September) +
+ +
1995
+
    +
  • Linear Logic and Applications Meeting in Cambridge (16 - 18 October) +
+
+

+ +Last modified: Mon Jul 11 14:49:50 CEST 2011 + +[Validate this page.] + +