src/HOL/Main.thy
changeset 74101 d804e93ae9ff
parent 73691 2f9877db82a1
child 74102 0572c733d12d
--- a/src/HOL/Main.thy	Sun Aug 01 23:18:13 2021 +0200
+++ b/src/HOL/Main.thy	Mon Aug 02 10:01:06 2021 +0000
@@ -71,4 +71,6 @@
   "_SUP1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3\<Squnion>_./ _)" [0, 10] 10)
   "_SUP"      :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b"  ("(3\<Squnion>_\<in>_./ _)" [0, 0, 10] 10)
 
+thy_deps
+
 end