More modification needed for compilation
authorCezary Kaliszyk <kaliszyk@in.tum.de>
Tue, 23 Mar 2010 09:34:32 +0100
changeset 1604 5ab97f43ec24
parent 1603 2b367c80c0d7
child 1605 d46a32cfcd89
More modification needed for compilation
Nominal/ExLF.thy
Nominal/ExLetRec.thy
Nominal/ExPS3.thy
Nominal/ExPS6.thy
Nominal/LFex.thy
Nominal/ROOT.ML
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/Nominal/ExLF.thy	Tue Mar 23 09:34:32 2010 +0100
@@ -0,0 +1,27 @@
+theory ExLF
+imports "Parser"
+begin
+
+atom_decl name
+atom_decl ident
+
+nominal_datatype kind =
+    Type
+  | KPi "ty" n::"name" k::"kind" bind n in k
+and ty =
+    TConst "ident"
+  | TApp "ty" "trm"
+  | TPi "ty" n::"name" t::"ty" bind n in t
+and trm =
+    Const "ident"
+  | Var "name"
+  | App "trm" "trm"
+  | Lam "ty" n::"name" t::"trm" bind n in t
+
+thm kind_ty_trm.supp
+
+end
+
+
+
+
--- a/Nominal/ExLetRec.thy	Tue Mar 23 09:21:43 2010 +0100
+++ b/Nominal/ExLetRec.thy	Tue Mar 23 09:34:32 2010 +0100
@@ -1,4 +1,4 @@
-theory ExLet
+theory ExLetRec
 imports "Parser"
 begin
 
--- a/Nominal/ExPS3.thy	Tue Mar 23 09:21:43 2010 +0100
+++ b/Nominal/ExPS3.thy	Tue Mar 23 09:34:32 2010 +0100
@@ -29,7 +29,8 @@
 thm exp_pat3.perm
 thm exp_pat3.induct
 thm exp_pat3.distinct
-thm exp_pat3.fv[simplified exp_pat3.supp]
+thm exp_pat3.fv
+thm exp_pat3.supp (* The bindings are too complicated *)
 
 end
 
--- a/Nominal/ExPS6.thy	Tue Mar 23 09:21:43 2010 +0100
+++ b/Nominal/ExPS6.thy	Tue Mar 23 09:34:32 2010 +0100
@@ -6,6 +6,9 @@
 
 atom_decl name
 
+(* The binding structure is too complicated, so we cannot show equivalence *)
+ML {* val _ = cheat_equivp := true *}
+
 ML {* val _ = recursive := false  *}
 nominal_datatype exp6 =
   EVar name
@@ -28,6 +31,7 @@
 thm exp6_pat6.perm
 thm exp6_pat6.induct
 thm exp6_pat6.distinct
+thm exp6_pat6.supp
 
 end
 
--- a/Nominal/LFex.thy	Tue Mar 23 09:21:43 2010 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,27 +0,0 @@
-theory LFex
-imports "Parser"
-begin
-
-atom_decl name
-atom_decl ident
-
-nominal_datatype kind =
-    Type
-  | KPi "ty" n::"name" k::"kind" bind n in k
-and ty =
-    TConst "ident"
-  | TApp "ty" "trm"
-  | TPi "ty" n::"name" t::"ty" bind n in t
-and trm =
-    Const "ident"
-  | Var "name"
-  | App "trm" "trm"
-  | Lam "ty" n::"name" t::"trm" bind n in t
-
-thm kind_ty_trm.supp
-
-end
-
-
-
-
--- a/Nominal/ROOT.ML	Tue Mar 23 09:21:43 2010 +0100
+++ b/Nominal/ROOT.ML	Tue Mar 23 09:34:32 2010 +0100
@@ -5,24 +5,17 @@
     "Nominal2_Eqvt",
     "Nominal2_Atoms",
     "Nominal2_Supp",
-    "Test"]
-
-(*
-no_document use_thys
-   ["Nominal2_Base",
-    "Nominal2_Eqvt",
-    "Nominal2_Atoms",
-    "Nominal2_Supp",
-    "Test",
-    "Term1",
-    "Term2",
-    "Term3",
-    "Term4",
-    "Term5",
-    "Term6",
-    "Term7",
-    "Term8",
-    "Term9",
-    "TySch",
-    "LFex"];
-*)
\ No newline at end of file
+    "ExLam",
+    "ExLF",
+    "Ex1",
+    "Ex1rec",
+    "Ex2",
+    "Ex3",
+    "ExLet",
+    "ExLetRec",
+    "ExTySch",
+    "ExLeroy"
+(*  "ExCoreHaskell", *)
+(*  "ExPS3", *)
+(*  "ExPS6", *)
+    ];