redundant since c6714a9562ae
authortraytel
Wed, 12 Jul 2017 07:52:35 +0200
changeset 66273 a5a24e1a6d6f
parent 66272 c6714a9562ae
child 66274 be8d3819c21c
redundant since c6714a9562ae
src/HOL/Library/Finite_Map.thy
--- a/src/HOL/Library/Finite_Map.thy	Tue Jul 11 21:36:42 2017 +0200
+++ b/src/HOL/Library/Finite_Map.thy	Wed Jul 12 07:52:35 2017 +0200
@@ -646,22 +646,6 @@
       rel: fmrel
   by auto
 
-text \<open>
-  Unfortunately, @{command lift_bnf} doesn't register the definitional theorems. We're doing it
-  manually below.
-\<close>
-
-local_setup \<open>fn lthy =>
-  let
-    val SOME bnf = BNF_Def.bnf_of lthy @{type_name fmap}
-  in
-    lthy
-    |> Local_Theory.note ((@{binding fmmap_def}, []), [BNF_Def.map_def_of_bnf bnf]) |> #2
-    |> Local_Theory.note ((@{binding fmran'_def}, []), BNF_Def.set_defs_of_bnf bnf) |> #2
-    |> Local_Theory.note ((@{binding fmrel_def}, []), [BNF_Def.rel_def_of_bnf bnf]) |> #2
-  end
-\<close>
-
 declare fmap.pred_mono[mono]
 
 context includes lifting_syntax begin