updated
authorChristian Urban <christian.urban@kcl.ac.uk>
Mon, 24 Jul 2023 09:46:42 +0100
changeset 638 bc23b95d3b2d
parent 637 eb530e39145d
child 639 88dcf2f5c2dd
updated
Nominal/users.html
--- a/Nominal/users.html	Sun Jul 09 08:56:24 2023 +0100
+++ b/Nominal/users.html	Mon Jul 24 09:46:42 2023 +0100
@@ -165,23 +165,20 @@
 proved the correctness of a GHC compiler transformation using Nominal2.
 This work appeared at the
 <A HREF="https://www.haskell.org/haskell-symposium/2015/">Haskell Symposium 2015</A>.
-</ul>
-</P>
 
-
-<H3>Entries in the Archive of Formal Proofs (AFP) using Nominal Isabelle</H3>
-
-<ul>
 <li>
-<A HREF="https://www.cl.cam.ac.uk/~mpew2/">Mark Wassell</A>, Alasdair
-Armstrong, Neel Krishnaswami and Peter Sewell mechanised the
-Metatheory for the MiniSail ISA Specification Language using Nominal
-Isabelle. They needed Nominal Isabelle for handling binding.  The AFP
-entry
-is <a href="https://www.isa-afp.org/entries/MiniSail.html">here</a>.
-This work appeared in the Proceedings of the 48th International
-Symposium on Microarchitecture MICRO-48 (2015) and at the Automated
-Reasoning Workshop (ARW 2018).
+  <A HREF="https://www.isa-afp.org/authors/brun">Matthias Brun</A> and
+  <A HREF="https://traytel.bitbucket.io/">Dmitriy Traytel</A> formalised
+  Generic Authenticated Data Structures using Nominal Isabelle.
+  The AFP entry is <a href="https://www.isa-afp.org/entries/Modal_Logics_for_NTS.html">here</a>.
+  This work appeared in the Proceedings of the International Conference on Concurrency Theory (CONCUR 2015).  
+
+<li>
+  <A HREF="https://www.isa-afp.org/authors/weber/">Tjark Weber</A> et al formalise a uniform
+  semantic substrate for a wide variety of process calculi where states and action labels can be from
+  arbitrary nominal sets. This includes a Hennessy-Milner logic for these systems.
+  The AFP entry is <a href="https://www.isa-afp.org/entries/Modal_Logics_for_NTS.html">here</a>.
+  This work appeared in the Proceedings of the International Conference on Concurrency Theory (CONCUR 2015).
 
 <li>
   <A HREF="https://www.andreipopescu.uk">Andrei Popescu</A> and
@@ -200,17 +197,67 @@
   The AFP entry is <a href="https://www.isa-afp.org/entries/LambdaAuth.html">here</a>.
   This work appeared in the Proceedings of International Conference on Interactive Theorem Proving (ITP 2019).
 
+
 <li>
-  <A HREF="https://www.isa-afp.org/authors/brun">Matthias Brun</A> and
-  <A HREF="https://traytel.bitbucket.io/">Dmitriy Traytel</A> formalised
-  Generic Authenticated Data Structures using Nominal Isabelle.
-  The AFP entry is <a href="https://www.isa-afp.org/entries/Modal_Logics_for_NTS.html">here</a>.
-  This work appeared in the Proceedings of the International Conference on Concurrency Theory (CONCUR 2015).  
+  <A HREF="https://www.andreipopescu.uk">Andrei Popescu</A> and
+  <A HREF="https://traytel.bitbucket.io/">Dmitriy Traytel</A>
+  formalise Robinson Arithmetic. This includes unary term-for-var substitution for two syntactic
+  categories (terms and formulas) and proves 15 delicate theorems: compositionality of substitution
+  w.r.t. itself, freshness, constructors. The AFP entry is
+  <a href="https://www.isa-afp.org/entries/Robinson_Arithmetic.html">here</a>.
+  This work appeared in the Proceedings of the International Conference on Automated Deduction (CADE 2019).  
+  
 </ul>
 </P>
 
 
+<H3>Entries in the Archive of Formal Proofs (AFP) using Nominal Isabelle</H3>
 
+<ul>
+<li>
+<A HREF="http://www.joachim-breitner.de/blog/" target="_top">Joachim Breitner</A>
+proved the correctness of a GHC compiler transformation using Nominal2.
+The AFP
+entry
+is <a href="https://www.isa-afp.org/entries/Call_Arity.html">here</a>.
+This work appeared at the
+<A HREF="https://www.haskell.org/haskell-symposium/2015/">Haskell Symposium 2015</A>.  
+
+  
+<li>
+<A HREF="https://www.cl.cam.ac.uk/~mpew2/">Mark Wassell</A>, Alasdair
+Armstrong, Neel Krishnaswami and Peter Sewell mechanised the
+Metatheory for the MiniSail ISA Specification Language using Nominal
+Isabelle. They needed Nominal Isabelle for handling binding.  The AFP
+entry
+is <a href="https://www.isa-afp.org/entries/MiniSail.html">here</a>.
+This work appeared in the Proceedings of the 48th International
+Symposium on Microarchitecture MICRO-48 (2015) and at the Automated
+Reasoning Workshop (ARW 2018).
+
+
+<li>
+  <A HREF="https://www.isa-afp.org/authors/felgenhauer/">Bertram Felgenhauer</A> et al formalise the
+  Z property introduced by Dehornoy and van Oostrom using Nominal 2.
+  The AFP entry is <a href="https://www.isa-afp.org/entries/Rewriting_Z.html">here</a>.
+
+
+  
+
+</ul>
+</P>
+
+<H3>Entries in the Archive of Formal that had to work around the current limitations of Nominal</H3>
+
+<ul>
+<li>
+<A HREF="https://www.isa-afp.org/authors/felgenhauer">Bertram Felgenhauer</A>
+formalised a higher-order term algebra, generalizing the notions of free variables, matching, and substitution.
+The Nominal framework provides support for reasoning over fresh names, but unfortunately,
+its definitions are not executable. The AFP entry
+is <a href="https://www.isa-afp.org/entries/Higher_Order_Terms.html">here</a>.
+</ul>
+</P>
 
 </TABLE>
 </CENTER>