Merge
authorcek@localhost.localdomain
Sat, 24 Oct 2009 16:15:33 +0200
changeset 176 3a8978c335f0
parent 175 f7602653dddd (current diff)
parent 174 09048a951dca (diff)
child 177 bdfe4388955d
child 178 945786a68ec6
Merge
FSet.thy
--- a/FSet.thy	Sat Oct 24 16:15:58 2009 +0200
+++ b/FSet.thy	Sat Oct 24 16:15:33 2009 +0200
@@ -14,18 +14,11 @@
 quotient qt = "t" / "Rt"
     by (rule t_eq)
 
-setup {*
-  maps_update @{type_name "list"} {mapfun = @{const_name "map"},      relfun = @{const_name "LIST_REL"}} #>
-  maps_update @{type_name "*"}    {mapfun = @{const_name "prod_fun"}, relfun = @{const_name "prod_rel"}} #>
-  maps_update @{type_name "fun"}  {mapfun = @{const_name "fun_map"},  relfun = @{const_name "FUN_REL"}}
-*}
-
-
 ML {*
 get_fun repF @{typ t} @{typ qt} @{context} @{typ "((((qt \<Rightarrow> qt) \<Rightarrow> qt) \<Rightarrow> qt) list) * nat"}
  |> fst
  |> Syntax.string_of_term @{context}
- |> writeln
+ |> writeln*)
 *}
 
 ML {*
--- a/QuotMain.thy	Sat Oct 24 16:15:58 2009 +0200
+++ b/QuotMain.thy	Sat Oct 24 16:15:33 2009 +0200
@@ -158,6 +158,12 @@
 use "quotient.ML"
 
 (* mapfuns for some standard types *)
+setup {*
+  maps_update @{type_name "list"} {mapfun = @{const_name "map"},      relfun = @{const_name "LIST_REL"}} #>
+  maps_update @{type_name "*"}    {mapfun = @{const_name "prod_fun"}, relfun = @{const_name "prod_rel"}} #>
+  maps_update @{type_name "fun"}  {mapfun = @{const_name "fun_map"},  relfun = @{const_name "FUN_REL"}}
+*}
+
 
 ML {* quotdata_lookup @{theory} *}
 setup {* quotdata_update_thy (@{typ nat}, @{typ bool}, @{term "True"})*}