src/Pure/pure_thy.ML
changeset 79336 032a31db4c6f
parent 79120 45b2171e9e03
child 80753 66893c47500d
--- a/src/Pure/pure_thy.ML	Fri Dec 22 17:19:08 2023 +0100
+++ b/src/Pure/pure_thy.ML	Fri Dec 22 21:03:16 2023 +0100
@@ -225,7 +225,7 @@
     (qualify (Binding.make ("sort_constraint", \<^here>)), typ "'a itself \<Rightarrow> prop", NoSyn),
     (qualify (Binding.make ("conjunction", \<^here>)), typ "prop \<Rightarrow> prop \<Rightarrow> prop", NoSyn)]
   #> Sign.local_path
-  #> (Global_Theory.add_defs false o map Thm.no_attributes)
+  #> fold (snd oo Global_Theory.add_def)
    [(Binding.make ("prop_def", \<^here>),
       prop "(CONST Pure.prop :: prop \<Rightarrow> prop) (A::prop) \<equiv> A::prop"),
     (Binding.make ("term_def", \<^here>),
@@ -234,7 +234,7 @@
       prop "(CONST Pure.sort_constraint :: 'a itself \<Rightarrow> prop) (CONST Pure.type :: 'a itself) \<equiv>\
       \ (CONST Pure.term :: 'a itself \<Rightarrow> prop) (CONST Pure.type :: 'a itself)"),
     (Binding.make ("conjunction_def", \<^here>),
-      prop "(A &&& B) \<equiv> (\<And>C::prop. (A \<Longrightarrow> B \<Longrightarrow> C) \<Longrightarrow> C)")] #> snd
+      prop "(A &&& B) \<equiv> (\<And>C::prop. (A \<Longrightarrow> B \<Longrightarrow> C) \<Longrightarrow> C)")]
   #> fold (#2 oo Thm.add_axiom_global) Theory.equality_axioms);
 
 end;